Loogle!
Result
Found 2603 declarations mentioning String. Of these, 169 have a name containing "Name".
- Lean.Name.mkSimple π Init.Prelude
(s : String) : Lean.Name - Lean.Name.mkStr1 π Init.Prelude
(sβ : String) : Lean.Name - Lean.Name.mkStr π Init.Prelude
(p : Lean.Name) (s : String) : Lean.Name - Lean.Name.mkStr2 π Init.Prelude
(sβ sβ : String) : Lean.Name - Lean.Name.str π Init.Prelude
(pre : Lean.Name) (str : String) : Lean.Name - Lean.Name.mkStr3 π Init.Prelude
(sβ sβ sβ : String) : Lean.Name - Lean.Name.mkStr4 π Init.Prelude
(sβ sβ sβ sβ : String) : Lean.Name - Lean.Name.mkStr5 π Init.Prelude
(sβ sβ sβ sβ sβ : String) : Lean.Name - Lean.Macro.resolveGlobalName π Init.Prelude
(n : Lean.Name) : Lean.MacroM (List (Lean.Name Γ List String)) - Lean.Name.mkStr6 π Init.Prelude
(sβ sβ sβ sβ sβ sβ : String) : Lean.Name - Lean.Name.mkStr7 π Init.Prelude
(sβ sβ sβ sβ sβ sβ sβ : String) : Lean.Name - Lean.Macro.Methods.resolveGlobalName π Init.Prelude
(self : Lean.Macro.Methods) : Lean.Name β Lean.MacroM (List (Lean.Name Γ List String)) - Lean.Name.mkStr8 π Init.Prelude
(sβ sβ sβ sβ sβ sβ sβ sβ : String) : Lean.Name - Lean.Name.str.sizeOf_spec π Init.SizeOf
(p : Lean.Name) (s : String) : sizeOf (p.str s) = 1 + sizeOf p + sizeOf s - Lean.Name.str.injEq π Init.Core
(pre : Lean.Name) (str : String) (preβ : Lean.Name) (strβ : String) : (pre.str str = preβ.str strβ) = (pre = preβ β§ str = strβ) - String.toName π Init.Meta
(s : String) : Lean.Name - Lean.Name.appendAfter π Init.Meta
(n : Lean.Name) (suffix : String) : Lean.Name - Lean.Name.appendBefore π Init.Meta
(n : Lean.Name) (pre : String) : Lean.Name - Lean.Syntax.decodeNameLit π Init.Meta
(s : String) : Option Lean.Name - Lean.Name.toStringWithSep.maybeEscape π Init.Meta
(escape : Bool) (s : String) (force : Bool) : String - Lean.Syntax.mkNameLit π Init.Meta
(val : String) (info : Lean.SourceInfo := Lean.SourceInfo.none) : Lean.NameLit - Lean.Name.escapePart π Init.Meta
(s : String) (force : Bool := false) : Option String - Lean.Name.toStringWithSep π Init.Meta
(sep : String) (escape : Bool) (n : Lean.Name) (isToken : String β Bool := fun x => false) : String - Lean.Name.toString π Init.Meta
(n : Lean.Name) (escape : Bool := true) (isToken : String β Bool := fun x => false) : String - System.FilePath.fileName π Init.System.FilePath
(p : System.FilePath) : Option String - System.FilePath.withFileName π Init.System.FilePath
(p : System.FilePath) (fname : String) : System.FilePath - IO.FS.DirEntry.fileName π Init.System.IO
(self : IO.FS.DirEntry) : String - Std.Time.TimeZone.name π Std.Time.Zoned.TimeZone
(self : Std.Time.TimeZone) : String - Std.Net.InterfaceAddress.name π Std.Net.Addr
(self : Std.Net.InterfaceAddress) : String - Std.Internal.UV.System.osGetHostname π Std.Internal.UV.System
: IO String - Std.Internal.UV.System.GroupInfo.groupname π Std.Internal.UV.System
(self : Std.Internal.UV.System.GroupInfo) : String - Std.Internal.UV.System.PasswdInfo.username π Std.Internal.UV.System
(self : Std.Internal.UV.System.PasswdInfo) : String - Std.Internal.UV.System.UnameInfo.machine π Std.Internal.UV.System
(self : Std.Internal.UV.System.UnameInfo) : String - Std.Internal.UV.System.UnameInfo.release π Std.Internal.UV.System
(self : Std.Internal.UV.System.UnameInfo) : String - Std.Internal.UV.System.UnameInfo.sysname π Std.Internal.UV.System
(self : Std.Internal.UV.System.UnameInfo) : String - Std.Internal.UV.System.UnameInfo.version π Std.Internal.UV.System
(self : Std.Internal.UV.System.UnameInfo) : String - Std.Internal.UV.System.UnameInfo.mk π Std.Internal.UV.System
(sysname release version machine : String) : Std.Internal.UV.System.UnameInfo - Std.Internal.UV.System.UnameInfo.mk.injEq π Std.Internal.UV.System
(sysname release version machine sysnameβ releaseβ versionβ machineβ : String) : ({ sysname := sysname, release := release, version := version, machine := machine } = { sysname := sysnameβ, release := releaseβ, version := versionβ, machine := machineβ }) = (sysname = sysnameβ β§ release = releaseβ β§ version = versionβ β§ machine = machineβ) - Std.Internal.UV.System.UnameInfo.mk.sizeOf_spec π Std.Internal.UV.System
(sysname release version machine : String) : sizeOf { sysname := sysname, release := release, version := version, machine := machine } = 1 + sizeOf sysname + sizeOf release + sizeOf version + sizeOf machine - Std.Internal.UV.DNS.getNameInfo π Std.Internal.UV.DNS
(host : Std.Net.SocketAddress) : IO (IO.Promise (Except IO.Error (String Γ String))) - Std.Internal.IO.Async.DNS.NameInfo.host π Std.Internal.Async.DNS
(self : Std.Internal.IO.Async.DNS.NameInfo) : String - Std.Internal.IO.Async.DNS.NameInfo.service π Std.Internal.Async.DNS
(self : Std.Internal.IO.Async.DNS.NameInfo) : String - Std.Internal.IO.Async.DNS.NameInfo.mk π Std.Internal.Async.DNS
(host service : String) : Std.Internal.IO.Async.DNS.NameInfo - Std.Internal.IO.Async.DNS.NameInfo.mk.injEq π Std.Internal.Async.DNS
(host service hostβ serviceβ : String) : ({ host := host, service := service } = { host := hostβ, service := serviceβ }) = (host = hostβ β§ service = serviceβ) - Std.Internal.IO.Async.DNS.NameInfo.mk.sizeOf_spec π Std.Internal.Async.DNS
(host service : String) : sizeOf { host := host, service := service } = 1 + sizeOf host + sizeOf service - Std.Internal.IO.Async.System.getHostName π Std.Internal.Async.System
: IO String - Std.Internal.IO.Async.System.GroupInfo.groupName π Std.Internal.Async.System
(self : Std.Internal.IO.Async.System.GroupInfo) : String - Std.Internal.IO.Async.System.OSInfo.name π Std.Internal.Async.System
(self : Std.Internal.IO.Async.System.OSInfo) : String - Std.Internal.IO.Async.System.SystemUser.username π Std.Internal.Async.System
(self : Std.Internal.IO.Async.System.SystemUser) : String - Lean.Name.getString! π Lean.Data.Name
: Lean.Name β String - Lean.Name.eqStr π Lean.Data.Name
: Lean.Name β String β Bool - Lean.Name.isInternalDetail.matchPrefix π Lean.Data.Name
(s pre : String) : Bool - Lean.Name.anyS π Lean.Data.Name
(n : Lean.Name) (f : String β Bool) : Bool - Lean.NamePart.str π Lean.Data.NameTrie
(s : String) : Lean.NamePart - Lean.NamePart.str.injEq π Lean.Data.NameTrie
(s sβ : String) : (Lean.NamePart.str s = Lean.NamePart.str sβ) = (s = sβ) - Lean.NamePart.str.sizeOf_spec π Lean.Data.NameTrie
(s : String) : sizeOf (Lean.NamePart.str s) = 1 + sizeOf s - Lean.Name.fromJson? π Lean.Data.Json.FromToJson
(j : Lean.Json) : Except String Lean.Name - Lean.NameMap.fromJson? π Lean.Data.Json.FromToJson
{Ξ± : Type} [Lean.FromJson Ξ±] : Lean.Json β Except String (Lean.NameMap Ξ±) - Lean.Expr.ctorName π Lean.Expr
: Lean.Expr β String - Lean.Server.instRpcEncodableWithRpcRefOfTypeName.rpcDecode π Lean.Server.Rpc.Basic
{Ξ± : Type} [TypeName Ξ±] (j : Lean.Json) : ExceptT String (ReaderT Lean.Server.RpcObjectStore Id) (Lean.Server.WithRpcRef Ξ±) - Lean.errorNameSuffix π Lean.Message
: String - Lean.BaseMessage.fileName π Lean.Message
{Ξ± : Type u} (self : Lean.BaseMessage Ξ±) : String - Lean.ErrorExplanation.CodeInfo.parse.namedAttr π Lean.ErrorExplanation
: Std.Internal.Parsec.String.Parser (String Γ String) - Lean.MonadLog.getFileName π Lean.Log
{m : Type β Type} [self : Lean.MonadLog m] : m String - Lean.ResolveName.resolveGlobalName π Lean.ResolveName
(env : Lean.Environment) (ns : Lean.Name) (openDecls : List Lean.OpenDecl) (id : Lean.Name) : List (Lean.Name Γ List String) - Lean.ensureReservedNameAvailable π Lean.ResolveName
{m : Type β Type} [Monad m] [Lean.MonadEnv m] [Lean.MonadError m] (declName : Lean.Name) (suffix : String) : m Unit - Lean.ResolveName.resolveGlobalName.loop π Lean.ResolveName
(env : Lean.Environment) (ns : Lean.Name) (openDecls : List Lean.OpenDecl) (extractionResult : Lean.MacroScopesView) (id : Lean.Name) (projs : List String) : List (Lean.Name Γ List String) - Lean.resolveGlobalName π Lean.ResolveName
{m : Type β Type} [Monad m] [Lean.MonadResolveName m] [Lean.MonadEnv m] (id : Lean.Name) : m (List (Lean.Name Γ List String)) - Lean.resolveLocalName π Lean.ResolveName
{m : Type β Type} [Monad m] [Lean.MonadResolveName m] [Lean.MonadEnv m] [Lean.MonadLCtx m] (n : Lean.Name) : m (Option (Lean.Expr Γ List String)) - Lean.resolveLocalName.loop π Lean.ResolveName
{m : Type β Type} [Monad m] [Lean.MonadResolveName m] [Lean.MonadEnv m] (view : Lean.MacroScopesView) (findLocalDecl? : Lean.MacroScopesView β Bool β Option Lean.LocalDecl) (n : Lean.Name) (projs : List String) (globalDeclFound : Bool) : m (Option (Lean.Expr Γ List String)) - Lean.Parser.InputContext.fileName π Lean.Parser.Types
(self : Lean.Parser.InputContext) : String - Lean.Core.Context.fileName π Lean.CoreM
(self : Lean.Core.Context) : String - Lean.Lsp.RenameFile.annotationId? π Lean.Data.Lsp.Basic
(self : Lean.Lsp.RenameFile) : Option String - Lean.Lsp.RenameFile.mk π Lean.Data.Lsp.Basic
(oldUri newUri : Lean.Lsp.DocumentUri) (options? : Option Lean.Lsp.CreateFile.Options) (annotationId? : Option String) : Lean.Lsp.RenameFile - Lean.Lsp.RenameFile.mk.injEq π Lean.Data.Lsp.Basic
(oldUri newUri : Lean.Lsp.DocumentUri) (options? : Option Lean.Lsp.CreateFile.Options) (annotationId? : Option String) (oldUriβ newUriβ : Lean.Lsp.DocumentUri) (options?β : Option Lean.Lsp.CreateFile.Options) (annotationId?β : Option String) : ({ oldUri := oldUri, newUri := newUri, options? := options?, annotationId? := annotationId? } = { oldUri := oldUriβ, newUri := newUriβ, options? := options?β, annotationId? := annotationId?β }) = (oldUri = oldUriβ β§ newUri = newUriβ β§ options? = options?β β§ annotationId? = annotationId?β) - Lean.Lsp.RenameFile.mk.sizeOf_spec π Lean.Data.Lsp.Basic
(oldUri newUri : Lean.Lsp.DocumentUri) (options? : Option Lean.Lsp.CreateFile.Options) (annotationId? : Option String) : sizeOf { oldUri := oldUri, newUri := newUri, options? := options?, annotationId? := annotationId? } = 1 + sizeOf oldUri + sizeOf newUri + sizeOf options? + sizeOf annotationId? - Lean.realizeGlobalName π Lean.ReservedNameAction
(id : Lean.Name) : Lean.CoreM (List (Lean.Name Γ List String)) - Lean.Elab.realizeGlobalNameWithInfos π Lean.Elab.InfoTree.Main
(ref : Lean.Syntax) (id : Lean.Name) : Lean.CoreM (List (Lean.Name Γ List String)) - Lean.getExternNameFor π Lean.Compiler.ExternAttr
(env : Lean.Environment) (backend fn : Lean.Name) : Option String - Lean.IR.getUnboxOpName π Lean.Compiler.IR.Basic
(t : Lean.IR.IRType) : String - Lean.Elab.InlayHintLabel.name π Lean.Elab.InfoTree.InlayHints
(n : String) : Lean.Elab.InlayHintLabel - Lean.Elab.InlayHintLabel.name.injEq π Lean.Elab.InfoTree.InlayHints
(n nβ : String) : (Lean.Elab.InlayHintLabel.name n = Lean.Elab.InlayHintLabel.name nβ) = (n = nβ) - Lean.Elab.InlayHintLabel.name.sizeOf_spec π Lean.Elab.InfoTree.InlayHints
(n : String) : sizeOf (Lean.Elab.InlayHintLabel.name n) = 1 + sizeOf n - Lean.Elab.Term.LVal.fieldName π Lean.Elab.Term
(ref : Lean.Syntax) (name : String) (suffix? : Option Lean.Name) (fullRef : Lean.Syntax) : Lean.Elab.Term.LVal - Lean.Elab.Term.MVarErrorInfo.logError.addArgName π Lean.Elab.Term
(mvarErrorInfo : Lean.Elab.Term.MVarErrorInfo) (msg : Lean.MessageData) (extra : String := "") : Lean.Elab.TermElabM Lean.MessageData - Lean.Elab.Term.resolveName.process π Lean.Elab.Term
(stx : Lean.Syntax) (n : Lean.Name) (explicitLevels : List Lean.Level) (candidates : List (Lean.Name Γ List String)) : Lean.Elab.TermElabM (List (Lean.Expr Γ List String)) - Lean.Elab.Term.resolveName π Lean.Elab.Term
(stx : Lean.Syntax) (n : Lean.Name) (preresolved : List Lean.Syntax.Preresolved) (explicitLevels : List Lean.Level) (expectedType? : Option Lean.Expr := none) : Lean.Elab.TermElabM (List (Lean.Expr Γ List String)) - Lean.Elab.Term.LVal.fieldName.injEq π Lean.Elab.Term
(ref : Lean.Syntax) (name : String) (suffix? : Option Lean.Name) (fullRef refβ : Lean.Syntax) (nameβ : String) (suffix?β : Option Lean.Name) (fullRefβ : Lean.Syntax) : (Lean.Elab.Term.LVal.fieldName ref name suffix? fullRef = Lean.Elab.Term.LVal.fieldName refβ nameβ suffix?β fullRefβ) = (ref = refβ β§ name = nameβ β§ suffix? = suffix?β β§ fullRef = fullRefβ) - Lean.Elab.Term.LVal.fieldName.sizeOf_spec π Lean.Elab.Term
(ref : Lean.Syntax) (name : String) (suffix? : Option Lean.Name) (fullRef : Lean.Syntax) : sizeOf (Lean.Elab.Term.LVal.fieldName ref name suffix? fullRef) = 1 + sizeOf ref + sizeOf name + sizeOf suffix? + sizeOf fullRef - Lean.Meta.isHCongrReservedNameSuffix π Lean.Meta.CongrTheorems
(s : String) : Bool - Lean.Meta.isEqnReservedNameSuffix π Lean.Meta.Eqns
(s : String) : Bool - Lean.Meta.mkEqLikeNameFor π Lean.Meta.Eqns
(env : Lean.Environment) (declName : Lean.Name) (suffix : String) : Lean.Name - Lean.Meta.declFromEqLikeName π Lean.Meta.Eqns
(env : Lean.Environment) (name : Lean.Name) : Option (Lean.Name Γ String) - Lean.Elab.Command.Context.fileName π Lean.Elab.Command
(self : Lean.Elab.Command.Context) : String - Lean.Lsp.LeanModule.name π Lean.Data.Lsp.Extra
(self : Lean.Lsp.LeanModule) : String - Lean.Lsp.CallHierarchyItem.name π Lean.Data.Lsp.LanguageFeatures
(self : Lean.Lsp.CallHierarchyItem) : String - Lean.Lsp.InlayHintLabel.name π Lean.Data.Lsp.LanguageFeatures
(n : String) : Lean.Lsp.InlayHintLabel - Lean.Lsp.ParameterInformationLabel.name π Lean.Data.Lsp.LanguageFeatures
(name : String) : Lean.Lsp.ParameterInformationLabel - Lean.Lsp.RenameParams.newName π Lean.Data.Lsp.LanguageFeatures
(self : Lean.Lsp.RenameParams) : String - Lean.Lsp.SemanticTokenModifier.names π Lean.Data.Lsp.LanguageFeatures
: Array String - Lean.Lsp.SemanticTokenType.names π Lean.Data.Lsp.LanguageFeatures
: Array String - Lean.Lsp.SymbolInformation.name π Lean.Data.Lsp.LanguageFeatures
(self : Lean.Lsp.SymbolInformation) : String - Lean.Lsp.RenameParams.mk π Lean.Data.Lsp.LanguageFeatures
(toTextDocumentPositionParams : Lean.Lsp.TextDocumentPositionParams) (newName : String) : Lean.Lsp.RenameParams - Lean.Lsp.SymbolInformation.containerName? π Lean.Data.Lsp.LanguageFeatures
(self : Lean.Lsp.SymbolInformation) : Option String - Lean.Lsp.DocumentSymbolAux.name π Lean.Data.Lsp.LanguageFeatures
{Self : Type} (self : Lean.Lsp.DocumentSymbolAux Self) : String - Lean.Lsp.InlayHintLabel.name.injEq π Lean.Data.Lsp.LanguageFeatures
(n nβ : String) : (Lean.Lsp.InlayHintLabel.name n = Lean.Lsp.InlayHintLabel.name nβ) = (n = nβ) - Lean.Lsp.ParameterInformationLabel.name.injEq π Lean.Data.Lsp.LanguageFeatures
(name nameβ : String) : (Lean.Lsp.ParameterInformationLabel.name name = Lean.Lsp.ParameterInformationLabel.name nameβ) = (name = nameβ) - Lean.Lsp.RenameParams.mk.injEq π Lean.Data.Lsp.LanguageFeatures
(toTextDocumentPositionParams : Lean.Lsp.TextDocumentPositionParams) (newName : String) (toTextDocumentPositionParamsβ : Lean.Lsp.TextDocumentPositionParams) (newNameβ : String) : ({ toTextDocumentPositionParams := toTextDocumentPositionParams, newName := newName } = { toTextDocumentPositionParams := toTextDocumentPositionParamsβ, newName := newNameβ }) = (toTextDocumentPositionParams = toTextDocumentPositionParamsβ β§ newName = newNameβ) - Lean.Lsp.InlayHintLabel.name.sizeOf_spec π Lean.Data.Lsp.LanguageFeatures
(n : String) : sizeOf (Lean.Lsp.InlayHintLabel.name n) = 1 + sizeOf n - Lean.Lsp.ParameterInformationLabel.name.sizeOf_spec π Lean.Data.Lsp.LanguageFeatures
(name : String) : sizeOf (Lean.Lsp.ParameterInformationLabel.name name) = 1 + sizeOf name - Lean.Lsp.RenameParams.mk.sizeOf_spec π Lean.Data.Lsp.LanguageFeatures
(toTextDocumentPositionParams : Lean.Lsp.TextDocumentPositionParams) (newName : String) : sizeOf { toTextDocumentPositionParams := toTextDocumentPositionParams, newName := newName } = 1 + sizeOf toTextDocumentPositionParams + sizeOf newName - Lean.Lsp.WorkspaceFolder.name π Lean.Data.Lsp.Workspace
(self : Lean.Lsp.WorkspaceFolder) : String - Lean.Lsp.ClientInfo.name π Lean.Data.Lsp.InitShutdown
(self : Lean.Lsp.ClientInfo) : String - Lean.Lsp.ServerInfo.name π Lean.Data.Lsp.InitShutdown
(self : Lean.Lsp.ServerInfo) : String - Lean.Lsp.RefInfo.ParentDecl.name π Lean.Data.Lsp.Internal
(self : Lean.Lsp.RefInfo.ParentDecl) : String - Lean.Widget.InteractiveGoal.userName? π Lean.Widget.InteractiveGoal
(self : Lean.Widget.InteractiveGoal) : Option String - Lean.Widget.InteractiveHypothesisBundle.names π Lean.Widget.InteractiveGoal
(self : Lean.Widget.InteractiveHypothesisBundle) : Array String - Lean.Elab.Tactic.Doc.TacticDoc.userName π Lean.Elab.Tactic.Doc
(self : Lean.Elab.Tactic.Doc.TacticDoc) : String - Lean.Linter.MissingDocs.lintNamed π Lean.Linter.MissingDocs
(stx : Lean.Syntax) (msg : String) : Lean.Elab.Command.CommandElabM Unit - Lean.NameMapAttributeImpl.descr π Batteries.Lean.NameMapAttribute
{Ξ± : Type} (self : Lean.NameMapAttributeImpl Ξ±) : String - Lean.NameMapAttributeImpl.mk π Batteries.Lean.NameMapAttribute
{Ξ± : Type} (name : Lean.Name) (ref : Lean.Name := by exact decl_name%) (descr : String) (add : Lean.Name β Lean.Syntax β Lean.AttrM Ξ±) : Lean.NameMapAttributeImpl Ξ± - Lean.NameMapAttributeImpl.mk.injEq π Batteries.Lean.NameMapAttribute
{Ξ± : Type} (name : Lean.Name) (ref : Lean.Name := by exact decl_name%) (descr : String) (add : Lean.Name β Lean.Syntax β Lean.AttrM Ξ±) (nameβ : Lean.Name) (refβ : Lean.Name := by exact decl_name%) (descrβ : String) (addβ : Lean.Name β Lean.Syntax β Lean.AttrM Ξ±) : ({ name := name, ref := ref, descr := descr, add := add } = { name := nameβ, ref := refβ, descr := descrβ, add := addβ }) = (name = nameβ β§ ref = refβ β§ descr = descrβ β§ add = addβ) - Lean.NameMapAttributeImpl.mk.sizeOf_spec π Batteries.Lean.NameMapAttribute
{Ξ± : Type} [SizeOf Ξ±] (name : Lean.Name) (ref : Lean.Name := by exact decl_name%) (descr : String) (add : Lean.Name β Lean.Syntax β Lean.AttrM Ξ±) : sizeOf { name := name, ref := ref, descr := descr, add := add } = 1 + sizeOf name + sizeOf ref + sizeOf descr - Lean.Elab.Command.mkNameFromParserSyntax.appendCatName π Lean.Elab.Syntax
(catName : Lean.Name) (str : String) : String - Lean.Elab.Command.mkNameFromParserSyntax.visit π Lean.Elab.Syntax
(stx : Lean.Syntax) (acc : String) : String - Lean.Widget.UserWidgetDefinition.name π Lean.Widget.UserWidget
(self : Lean.Widget.UserWidgetDefinition) : String - Lean.Widget.PanelWidgetInstance.name? π Lean.Widget.UserWidget
(self : Lean.Widget.PanelWidgetInstance) : Option String - Lean.Elab.Command.NameGen.mkBaseName π Lean.Elab.DeclNameGen
(e : Lean.Expr) : Lean.Elab.Command.NameGen.MkNameMβ String - Lean.Elab.Command.NameGen.mkBaseNameWithSuffix π Lean.Elab.DeclNameGen
(pre : String) (type : Lean.Expr) : Lean.MetaM Lean.Name - Lean.Elab.Command.NameGen.mkBaseNameWithSuffix' π Lean.Elab.DeclNameGen
(pre : String) (binders : Array Lean.Syntax) (type : Lean.Syntax) : Lean.Elab.TermElabM Lean.Name - Lean.Name.lastComponentAsString π Mathlib.Lean.Expr.Basic
: Lean.Name β String - Lean.Name.updateLast π Mathlib.Lean.Expr.Basic
(f : String β String) : Lean.Name β Lean.Name - Simps.Config.nameStem π Mathlib.Tactic.Simps.Basic
(self : Simps.Config) : Option String - ToAdditive.guessName π Mathlib.Tactic.ToAdditive.Frontend
: String β String - ToAdditive.nameDict π Mathlib.Tactic.ToAdditive.Frontend
: String β List String - ToAdditive.applyNameDict π Mathlib.Tactic.ToAdditive.Frontend
: List String β List String - ToAdditive.endCapitalNames π Mathlib.Tactic.ToAdditive.Frontend
: Std.TreeMap String (List String) compare - Lean.Xml.Parser.EncName π Lean.Data.Xml.Parser
: Std.Internal.Parsec.String.Parser String - Lean.Xml.Parser.Name π Lean.Data.Xml.Parser
: Std.Internal.Parsec.String.Parser String - Lean.mkModuleInitializationFunctionName π Lean.Compiler.NameMangling
(moduleName : Lean.Name) : String - Lean.Name.mangle π Lean.Compiler.NameMangling
(n : Lean.Name) (pre : String := "l_") : String - Lean.IR.EmitC.toCInitName π Lean.Compiler.IR.EmitC
(n : Lean.Name) : Lean.IR.EmitC.M String - Lean.IR.EmitC.toCName π Lean.Compiler.IR.EmitC
(n : Lean.Name) : Lean.IR.EmitC.M String - LLVM.Value.getName π Lean.Compiler.IR.LLVMBindings
{ctx : LLVM.Context} (value : LLVM.Value ctx) : BaseIO String - LLVM.getNamedFunction π Lean.Compiler.IR.LLVMBindings
{ctx : LLVM.Context} (m : LLVM.Module ctx) (name : String) : BaseIO (Option (LLVM.Value ctx)) - LLVM.getNamedGlobal π Lean.Compiler.IR.LLVMBindings
{ctx : LLVM.Context} (m : LLVM.Module ctx) (name : String) : BaseIO (Option (LLVM.Value ctx)) - Lean.IR.EmitLLVM.toCInitName π Lean.Compiler.IR.EmitLLVM
{llvmctx : LLVM.Context} (n : Lean.Name) : Lean.IR.EmitLLVM.M llvmctx String - Lean.IR.EmitLLVM.toCName π Lean.Compiler.IR.EmitLLVM
{llvmctx : LLVM.Context} (n : Lean.Name) : Lean.IR.EmitLLVM.M llvmctx String - Lean.Meta.Match.isCongrEqnReservedNameSuffix π Lean.Meta.Match.MatchEqs
(s : String) : Bool - Lean.Firefox.Thread.name π Lean.Util.Profiler
(self : Lean.Firefox.Thread) : String - Lean.Elab.Tactic.Omega.formatErrorMessage.varNameOf π Lean.Elab.Tactic.Omega.Frontend
(i : β) : String - Lean.Elab.Tactic.Omega.formatErrorMessage.varNames π Lean.Elab.Tactic.Omega.Frontend
(mask : Array Bool) : Lean.MetaM (Array String) - Lean.Server.Test.Runner.Client.Hyp.names π Lean.Server.Test.Runner
(self : Lean.Server.Test.Runner.Client.Hyp) : Array String - Lean.Linter.List.allowedArrayNames π Lean.Linter.List
: List String - Lean.Linter.List.allowedListNames π Lean.Linter.List
: List String - Lean.Linter.List.allowedVectorNames π Lean.Linter.List
: List String - Lean.Linter.List.stripBinderName π Lean.Linter.List
(s : String) : String - Aesop.LocalRuleSet.trace.printSimpSetName π Aesop.RuleSet
: Lean.Name β String - Aesop.StatsExtensionEntry.fileName π Aesop.Stats.Extension
(self : Aesop.StatsExtensionEntry) : String - Plausible.NamedBinder π Plausible.Testable
(_n : String) (p : Prop) : Prop - Plausible.NamedBinder.eq_1 π Plausible.Testable
(_n : String) (p : Prop) : Plausible.NamedBinder _n p = p - LeanSearchClient.SearchResult.name π LeanSearchClient.Syntax
(self : LeanSearchClient.SearchResult) : String - LeanSearchClient.SearchServer.name π LeanSearchClient.Syntax
(self : LeanSearchClient.SearchServer) : String - LeanSearchClient.LoogleMatch.name π LeanSearchClient.LoogleSyntax
(self : LeanSearchClient.LoogleMatch) : String - String.renameMetaVar π Mathlib.Tactic.Widget.SelectPanelUtils
(s : String) : String - Mathlib.Tactic.Polyrith.SageError.name π Mathlib.Tactic.Polyrith
(self : Mathlib.Tactic.Polyrith.SageError) : String - ProofWidgets.ExprPresentationData.userName π ProofWidgets.Presentation.Expr
(self : ProofWidgets.ExprPresentationData) : String - ProofWidgets.ExprPresenter.userName π ProofWidgets.Presentation.Expr
(self : ProofWidgets.ExprPresenter) : String - Loogle.Find.Arguments.namePats π Loogle.Find
(self : Loogle.Find.Arguments) : Array String
About
Loogle searches Lean and Mathlib definitions and theorems.
You can use Loogle from within the Lean4 VSCode language extension
using (by default) Ctrl-K Ctrl-S. You can also try the
#loogle
command from LeanSearchClient,
the CLI version, the Loogle
VS Code extension, the lean.nvim
integration or the Zulip bot.
Usage
Loogle finds definitions and lemmas in various ways:
By constant:
πReal.sin
finds all lemmas whose statement somehow mentions the sine function.By lemma name substring:
π"differ"
finds all lemmas that have"differ"
somewhere in their lemma name.By subexpression:
π_ * (_ ^ _)
finds all lemmas whose statements somewhere include a product where the second argument is raised to some power.The pattern can also be non-linear, as in
πReal.sqrt ?a * Real.sqrt ?a
If the pattern has parameters, they are matched in any order. Both of these will find
List.map
:
π(?a -> ?b) -> List ?a -> List ?b
πList ?a -> (?a -> ?b) -> List ?b
By main conclusion:
π|- tsum _ = _ * tsum _
finds all lemmas where the conclusion (the subexpression to the right of allβ
andβ
) has the given shape.As before, if the pattern has parameters, they are matched against the hypotheses of the lemma in any order; for example,
π|- _ < _ β tsum _ < tsum _
will findtsum_lt_tsum
even though the hypothesisf i < g i
is not the last.
If you pass more than one such search filter, separated by commas
Loogle will return lemmas which match all of them. The
search
π Real.sin, "two", tsum, _ * _, _ ^ _, |- _ < _ β _
would find all lemmas which mention the constants Real.sin
and tsum
, have "two"
as a substring of the
lemma name, include a product and a power somewhere in the type,
and have a hypothesis of the form _ < _
(if
there were any such lemmas). Metavariables (?a
) are
assigned independently in each filter.
The #lucky
button will directly send you to the
documentation of the first hit.
Source code
You can find the source code for this service at https://github.com/nomeata/loogle. The https://loogle.lean-lang.org/ service is provided by the Lean FRO.
This is Loogle revision ff04530
serving mathlib revision 5eb29c4