File tree Expand file tree Collapse file tree 1 file changed +0
-4
lines changed Expand file tree Collapse file tree 1 file changed +0
-4
lines changed Original file line number Diff line number Diff line change @@ -1079,10 +1079,6 @@ def synthesizeInstMVarCore (instMVar : MVarId) (maxResultSize? : Option Nat := n
1079
1079
else
1080
1080
throwError "failed to synthesize{indentExpr type}{extraErrorMsg}{useDiagnosticMsg}"
1081
1081
1082
- def mkCoeErrorMsg (f? : Option Expr) (errorMsgHeader? : Option String) (mvarId : MVarId) (expectedType e : Expr) : MetaM MessageData := do
1083
- throwTypeMismatchError errorMsgHeader? expectedType (← inferType e) e f?
1084
- m!"failed to create type class instance for{indentExpr (← mvarId.getDecl).type}"
1085
-
1086
1082
def mkCoe (expectedType : Expr) (e : Expr) (f? : Option Expr := none) (errorMsgHeader? : Option String := none)
1087
1083
(mkErrorMsg? : Option (MVarId → (expectedType e : Expr) → MetaM MessageData) := none)
1088
1084
(mkImmedErrorMsg? : Option ((errorMsg? : Option MessageData) → (expectedType e : Expr) → MetaM MessageData) := none) : TermElabM Expr := do
You can’t perform that action at this time.
0 commit comments