Documentation

Lean.ScopedEnvExtension

Instances For
    Instances For
      Equations
      • Lean.ScopedEnvExtension.instInhabitedScopedEntries = { default := { map := default } }
      structure Lean.ScopedEnvExtension.Descr (α β σ : Type) :
      • name : Lean.Name
      • mkInitial : IO σ
      • ofOLeanEntry : σαLean.ImportM β
      • toOLeanEntry : βα
      • addEntry : σβσ
      • finalizeImport : σσ
      Instances For
        Equations
        • One or more equations did not get rendered due to their size.
        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
            instance Lean.instInhabitedScopedEnvExtension {a✝ : Type} [Inhabited a✝] {a✝¹ a✝² : Type} :
            Inhabited (Lean.ScopedEnvExtension a✝ a✝¹ a✝²)
            Equations
            • Lean.instInhabitedScopedEnvExtension = { default := { descr := default, ext := default } }
            Instances For
              @[implemented_by Lean.registerScopedEnvExtensionUnsafe]
              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                Instances For
                  def Lean.ScopedEnvExtension.addScopedEntry {α β σ : Type} (ext : Lean.ScopedEnvExtension α β σ) (env : Lean.Environment) (namespaceName : Lean.Name) (b : β) :
                  Equations
                  Instances For
                    Instances For
                      def Lean.ScopedEnvExtension.addCore {α β σ : Type} (env : Lean.Environment) (ext : Lean.ScopedEnvExtension α β σ) (b : β) (kind : Lean.AttributeKind) (namespaceName : Lean.Name) :
                      Equations
                      Instances For
                        Equations
                        Instances For
                          Instances For
                            Instances For
                              def Lean.ScopedEnvExtension.modifyState {α β σ : Type} (ext : Lean.ScopedEnvExtension α β σ) (env : Lean.Environment) (f : σσ) :
                              Instances For
                                Instances For
                                  Equations
                                  • One or more equations did not get rendered due to their size.
                                  Instances For
                                    def Lean.activateScoped {m : TypeType} [Monad m] [Lean.MonadEnv m] [MonadLiftT (ST IO.RealWorld) m] (namespaceName : Lean.Name) :
                                    Equations
                                    • One or more equations did not get rendered due to their size.
                                    Instances For
                                      @[reducible, inline]
                                      Instances For
                                        • name : Lean.Name
                                        • addEntry : σασ
                                        • initial : σ
                                        • finalizeImport : σσ
                                        Instances For
                                          Equations
                                          • One or more equations did not get rendered due to their size.
                                          Instances For