File tree Expand file tree Collapse file tree 1 file changed +2
-1
lines changed Expand file tree Collapse file tree 1 file changed +2
-1
lines changed Original file line number Diff line number Diff line change @@ -9,6 +9,7 @@ import Lean.Parser.Term
9
9
import Lean.Meta.Structure
10
10
import Lean.Elab.App
11
11
import Lean.Elab.Binders
12
+ import Lean.PrettyPrinter
12
13
13
14
namespace Lean.Elab.Term.StructInst
14
15
@@ -433,7 +434,7 @@ private def expandParentFields (s : Struct) : TermElabM Struct := do
433
434
| { lhs := .fieldName ref fieldName :: _, .. } =>
434
435
addCompletionInfo <| CompletionInfo.fieldId ref fieldName (← getLCtx) s.structName
435
436
match findField? env s.structName fieldName with
436
- | none => throwErrorAt ref "'{fieldName}' is not a field of structure '{s.structName}'"
437
+ | none => throwErrorAt ref "'{fieldName}' is not a field of structure '{MessageData.ofConstName s.structName}'"
437
438
| some baseStructName =>
438
439
if baseStructName == s.structName then pure field
439
440
else match getPathToBaseStructure? env baseStructName s.structName with
You can’t perform that action at this time.
0 commit comments