Skip to content

Commit 58e134b

Browse files
committed
Extra removal
1 parent ada0c9f commit 58e134b

File tree

1 file changed

+0
-3
lines changed

1 file changed

+0
-3
lines changed

src/Lean/Elab/Tactic/BuiltinTactic.lean

Lines changed: 0 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -250,9 +250,6 @@ partial def evalChoiceAux (tactics : Array Syntax) (i : Nat) : TacticM Unit :=
250250

251251
@[builtin_tactic skip] def evalSkip : Tactic := fun _ => pure ()
252252

253-
@[builtin_tactic unknown] def evalUnknown : Tactic := fun stx => do
254-
addCompletionInfo <| CompletionInfo.tactic stx
255-
256253
@[builtin_tactic failIfSuccess] def evalFailIfSuccess : Tactic := fun stx =>
257254
Term.withoutErrToSorry <| withoutRecover do
258255
let tactic := stx[1]

0 commit comments

Comments
 (0)