Documentation

Lean.Elab.Import

@[reducible, inline]
Equations
Instances For
    Equations
    Instances For
      Equations
      Instances For
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          Equations
          Instances For
            @[reducible, inline]
            abbrev Lean.Elab.headerToImports (stx : HeaderSyntax) (includeInit : Bool := true) :
            Equations
            Instances For
              def Lean.Elab.processHeaderCore (startPos : String.Pos) (imports : Array Import) (isModule : Bool) (opts : Options) (messages : MessageLog) (inputCtx : Parser.InputContext) (trustLevel : UInt32 := 0) (plugins : Array System.FilePath := #[]) (leakEnv : Bool := false) (mainModule : Name := Name.anonymous) (arts : NameMap ImportArtifacts := ) :
              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                @[inline]
                def Lean.Elab.processHeader (header : HeaderSyntax) (opts : Options) (messages : MessageLog) (inputCtx : Parser.InputContext) (trustLevel : UInt32 := 0) (plugins : Array System.FilePath := #[]) (leakEnv : Bool := false) (mainModule : Name := Name.anonymous) :

                Elaborates the given header syntax into an environment.

                If mainModule is not given, Environment.setMainModule should be called manually. This is a backwards compatibility measure not compatible with the module system.

                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.Elab.printImports (input : String) (fileName : Option String) :
                    Equations
                    • One or more equations did not get rendered due to their size.
                    Instances For
                      def Lean.Elab.printImportSrcs (input : String) (fileName : Option String) :
                      Equations
                      • One or more equations did not get rendered due to their size.
                      Instances For