Skip to content

Commit

Permalink
chore: comment
Browse files Browse the repository at this point in the history
  • Loading branch information
Vtec234 authored Dec 12, 2023
1 parent fd5bff1 commit 93d22fa
Showing 1 changed file with 0 additions and 2 deletions.
2 changes: 0 additions & 2 deletions vscode-lean4/src/utils/converters.ts
Original file line number Diff line number Diff line change
Expand Up @@ -108,8 +108,6 @@ export function patchConverters(p2cConverter: Protocol2CodeConverter, c2pConvert
// eslint-disable-next-line @typescript-eslint/unbound-method
const oldP2cAsCodeAction = p2cConverter.asCodeAction
p2cConverter.asCodeAction = async function (item: ls.CodeAction | null | undefined, token?: code.CancellationToken) {
// if (item.diagnostics !== undefined) { result.diagnostics = asDiagnosticsSync(item.diagnostics); }
// if (item.edit !== undefined) { result.edit = await asWorkspaceEdit(item.edit, token); }
if (item === undefined || item === null) return undefined
if (item.edit || item.diagnostics) {
const result: code.CodeAction = await oldP2cAsCodeAction.apply(this, [item, token])
Expand Down

0 comments on commit 93d22fa

Please sign in to comment.