File tree Expand file tree Collapse file tree 3 files changed +3
-3
lines changed
Expand file tree Collapse file tree 3 files changed +3
-3
lines changed Original file line number Diff line number Diff line change @@ -52,7 +52,7 @@ def hasTrivialStructure? (declName : Name) : CoreM (Option TrivialStructureInfo)
5252 trivialStructureInfoExt.insert declName info?
5353 return info?
5454where fillCache : CoreM (Option TrivialStructureInfo) := do
55- if isRuntimeBultinType declName then return none
55+ if isRuntimeBuiltinType declName then return none
5656 let .inductInfo info ← getConstInfo declName | return none
5757 if info.isUnsafe || info.isRec then return none
5858 let [ctorName] := info.ctors | return none
Original file line number Diff line number Diff line change @@ -671,7 +671,7 @@ where
671671
672672 visitProjFn (projInfo : ProjectionFunctionInfo) (e : Expr) : M Arg := do
673673 let typeName := projInfo.ctorName.getPrefix
674- if isRuntimeBultinType typeName then
674+ if isRuntimeBuiltinType typeName then
675675 let numArgs := e.getAppNumArgs
676676 let arity := projInfo.numParams + 1
677677 if numArgs < arity then
Original file line number Diff line number Diff line change @@ -89,7 +89,7 @@ def builtinRuntimeTypes : Array Name := #[
8989/--
9090Return `true` iff `declName` is the name of a type with builtin support in the runtime.
9191-/
92- def isRuntimeBultinType (declName : Name) : Bool :=
92+ def isRuntimeBuiltinType (declName : Name) : Bool :=
9393 builtinRuntimeTypes.contains declName
9494
9595end Lean.Compiler.LCNF
You can’t perform that action at this time.
0 commit comments