Skip to content

Commit f31ef3f

Browse files
committed
remove unused function
1 parent 5a0249e commit f31ef3f

File tree

1 file changed

+0
-4
lines changed

1 file changed

+0
-4
lines changed

src/Lean/Elab/Term.lean

Lines changed: 0 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -1079,10 +1079,6 @@ def synthesizeInstMVarCore (instMVar : MVarId) (maxResultSize? : Option Nat := n
10791079
else
10801080
throwError "failed to synthesize{indentExpr type}{extraErrorMsg}{useDiagnosticMsg}"
10811081

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-
10861082
def mkCoe (expectedType : Expr) (e : Expr) (f? : Option Expr := none) (errorMsgHeader? : Option String := none)
10871083
(mkErrorMsg? : Option (MVarId → (expectedType e : Expr) → MetaM MessageData) := none)
10881084
(mkImmedErrorMsg? : Option ((errorMsg? : Option MessageData) → (expectedType e : Expr) → MetaM MessageData) := none) : TermElabM Expr := do

0 commit comments

Comments
 (0)