Documentation

Lean.DocString

def Lean.addBuiltinDocString (declName : Lake.Name) (docString : String) :
Equations
Instances For
    def Lean.addDocString {m : TypeType} [Lean.MonadEnv m] (declName : Lake.Name) (docString : String) :
    Equations
    Instances For
      def Lean.addDocString' {m : TypeType} [Monad m] [Lean.MonadEnv m] (declName : Lake.Name) (docString? : Option String) :
      Equations
      Instances For
        def Lean.findDocString? (env : Lean.Environment) (declName : Lake.Name) (includeBuiltin : optParam Bool true) :
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          structure Lean.ModuleDoc :
          Instances For
            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              def Lean.getDocStringText {m : TypeType} [Monad m] [Lean.MonadError m] [Lean.MonadRef m] (stx : Lean.TSyntax `Lean.Parser.Command.docComment) :
              Equations
              • One or more equations did not get rendered due to their size.
              Instances For