Built with doc-gen4, running Lean4. Bubbles () indicate interactive fragments: hover for details, tap to reveal contents. Use Ctrl+↑Ctrl+↓to navigate, Ctrl+🖱️to focus. On Mac, use Cmdinstead of Ctrl.
/-
Copyright (c) 2022 Gabriel Ebner. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Gabriel Ebner
-/
import Lean.Attributes

/-- Get the list of declarations tagged with the tag attribute `attr`. -/
def 
Lean.TagAttribute.getDecls: TagAttributeEnvironmentArray Name
Lean.TagAttribute.getDecls
(attr :
TagAttribute: Type
TagAttribute
) (env :
Environment: Type
Environment
) :
Array: Type ?u.6 → Type ?u.6
Array
Name: Type
Name
:= core <| attr.ext.
toEnvExtension: {α β σ : Type} → PersistentEnvExtension α β σEnvExtension (PersistentEnvExtensionState α σ)
toEnvExtension
.
getState: {σ : Type} → [inst : Inhabited σ] → EnvExtension σEnvironmentσ
getState
env where /-- Implementation of `TagAttribute.getDecls`. -/ core (st :
PersistentEnvExtensionState: TypeTypeType
PersistentEnvExtensionState
Name: Type
Name
NameSet: Type
NameSet
) :
Array: Type ?u.13 → Type ?u.13
Array
Name: Type
Name
:=
Id.run: {α : Type ?u.17} → Id αα
Id.run
do let mut
decls: ?m.38
decls
:= st.
state: {α σ : Type} → PersistentEnvExtensionState α σσ
state
.
toArray: {α : Type ?u.43} → {cmp : ααOrdering} → RBTree α cmpArray α
toArray
for
ds: ?m.143
ds
in st.
importedEntries: {α σ : Type} → PersistentEnvExtensionState α σArray (Array α)
importedEntries
do
decls: ?m.152
decls
:=
decls: ?m.149
decls
++
ds: ?m.143
ds
decls: ?m.326
decls