Documentation

Lean.ScopedEnvExtension

Instances For
    Instances For
      Instances For
        Instances For
          instance Lean.ScopedEnvExtension.instInhabitedStateStack {a✝ a✝¹ a✝² : Type} :
          Inhabited (StateStack a✝ a✝¹ a✝²)
          Equations
          structure Lean.ScopedEnvExtension.Descr (α β σ : Type) :
          • name : Name
          • mkInitial : IO σ
          • ofOLeanEntry : σαImportM β
          • toOLeanEntry : βα
          • addEntry : σβσ
          • finalizeImport : σσ
          Instances For
            Equations
            • One or more equations did not get rendered due to their size.
            def Lean.ScopedEnvExtension.mkInitial {α β σ : Type} (descr : Descr α β σ) :
            IO (StateStack α β σ)
            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              def Lean.ScopedEnvExtension.ScopedEntries.insert {β : Type} (scopedEntries : ScopedEntries β) (ns : Name) (b : β) :
              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                def Lean.ScopedEnvExtension.addImportedFn {α β σ : Type} (descr : Descr α β σ) (as : Array (Array (Entry α))) :
                ImportM (StateStack α β σ)
                Equations
                • One or more equations did not get rendered due to their size.
                Instances For
                  def Lean.ScopedEnvExtension.addEntryFn {α β σ : Type} (descr : Descr α β σ) (s : StateStack α β σ) (e : Entry β) :
                  StateStack α β σ
                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For
                    def Lean.ScopedEnvExtension.exportEntriesFn {α β σ : Type} (s : StateStack α β σ) :
                    Equations
                    Instances For
                      structure Lean.ScopedEnvExtension (α β σ : Type) :
                      Instances For
                        instance Lean.instInhabitedScopedEnvExtension {a✝ : Type} [Inhabited a✝] {a✝¹ a✝² : Type} :
                        Inhabited (ScopedEnvExtension a✝ a✝¹ a✝²)
                        Equations
                        unsafe def Lean.registerScopedEnvExtensionUnsafe {α β σ : Type} (descr : ScopedEnvExtension.Descr α β σ) :
                        Equations
                        • One or more equations did not get rendered due to their size.
                        Instances For
                          @[implemented_by Lean.registerScopedEnvExtensionUnsafe]
                          opaque Lean.registerScopedEnvExtension {α β σ : Type} (descr : ScopedEnvExtension.Descr α β σ) :
                          Equations
                          • One or more equations did not get rendered due to their size.
                          Instances For
                            Equations
                            • One or more equations did not get rendered due to their size.
                            Instances For
                              def Lean.ScopedEnvExtension.addEntry {α β σ : Type} (ext : ScopedEnvExtension α β σ) (env : Environment) (b : β) :
                              Equations
                              Instances For
                                def Lean.ScopedEnvExtension.addScopedEntry {α β σ : Type} (ext : ScopedEnvExtension α β σ) (env : Environment) (namespaceName : Name) (b : β) :
                                Equations
                                Instances For
                                  def Lean.ScopedEnvExtension.addLocalEntry {α β σ : Type} (ext : ScopedEnvExtension α β σ) (env : Environment) (b : β) :
                                  Equations
                                  • One or more equations did not get rendered due to their size.
                                  Instances For
                                    def Lean.ScopedEnvExtension.addCore {α β σ : Type} (env : Environment) (ext : ScopedEnvExtension α β σ) (b : β) (kind : AttributeKind) (namespaceName : Name) :
                                    Equations
                                    Instances For
                                      def Lean.ScopedEnvExtension.add {m : TypeType} {α β σ : Type} [Monad m] [MonadResolveName m] [MonadEnv m] (ext : ScopedEnvExtension α β σ) (b : β) (kind : AttributeKind := AttributeKind.global) :
                                      Equations
                                      Instances For
                                        def Lean.ScopedEnvExtension.getState {σ α β : Type} [Inhabited σ] (ext : ScopedEnvExtension α β σ) (env : Environment) :
                                        σ
                                        Equations
                                        • One or more equations did not get rendered due to their size.
                                        Instances For
                                          def Lean.ScopedEnvExtension.activateScoped {α β σ : Type} (ext : ScopedEnvExtension α β σ) (env : Environment) (namespaceName : Name) :
                                          Equations
                                          • One or more equations did not get rendered due to their size.
                                          Instances For
                                            def Lean.ScopedEnvExtension.modifyState {α β σ : Type} (ext : ScopedEnvExtension α β σ) (env : Environment) (f : σσ) :
                                            Equations
                                            • One or more equations did not get rendered due to their size.
                                            Instances For
                                              Equations
                                              • One or more equations did not get rendered due to their size.
                                              Instances For
                                                Equations
                                                • One or more equations did not get rendered due to their size.
                                                Instances For
                                                  def Lean.activateScoped {m : TypeType} [Monad m] [MonadEnv m] [MonadLiftT (ST IO.RealWorld) m] (namespaceName : Name) :
                                                  Equations
                                                  • One or more equations did not get rendered due to their size.
                                                  Instances For
                                                    @[reducible, inline]
                                                    Equations
                                                    Instances For
                                                      • name : Name
                                                      • addEntry : σασ
                                                      • initial : σ
                                                      • finalizeImport : σσ
                                                      Instances For
                                                        Equations
                                                        • One or more equations did not get rendered due to their size.
                                                        Instances For