We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent ada0c9f commit 58e134bCopy full SHA for 58e134b
src/Lean/Elab/Tactic/BuiltinTactic.lean
@@ -250,9 +250,6 @@ partial def evalChoiceAux (tactics : Array Syntax) (i : Nat) : TacticM Unit :=
250
251
@[builtin_tactic skip] def evalSkip : Tactic := fun _ => pure ()
252
253
-@[builtin_tactic unknown] def evalUnknown : Tactic := fun stx => do
254
- addCompletionInfo <| CompletionInfo.tactic stx
255
-
256
@[builtin_tactic failIfSuccess] def evalFailIfSuccess : Tactic := fun stx =>
257
Term.withoutErrToSorry <| withoutRecover do
258
let tactic := stx[1]
0 commit comments