Skip to content

Commit

Permalink
docs(tactic/interactive): Add tag debugging and doc mwe for `extr…
Browse files Browse the repository at this point in the history
  • Loading branch information
utensil and robertylewis committed Aug 6, 2020
1 parent ee7bb12 commit 224e0f8
Showing 1 changed file with 3 additions and 2 deletions.
5 changes: 3 additions & 2 deletions src/tactic/interactive.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1045,7 +1045,8 @@ do ls ← local_context,
partition_vars' (name_set.of_list $ ls.map expr.local_uniq_name) ls [] []

/--
Format the current goal as a stand-alone example. Useful for testing tactic.
Format the current goal as a stand-alone example. Useful for testing tactics
or creating [minimal working examples](https://leanprover-community.github.io/mwe.html).
* `extract_goal`: formats the statement as an `example` declaration
* `extract_goal my_decl`: formats the statement as a `lemma` or `def` declaration
Expand Down Expand Up @@ -1153,7 +1154,7 @@ add_tactic_doc
{ name := "extract_goal",
category := doc_category.tactic,
decl_names := [`tactic.interactive.extract_goal],
tags := ["goal management", "proof extraction"] }
tags := ["goal management", "proof extraction", "debugging"] }

/--
`inhabit α` tries to derive a `nonempty α` instance and then upgrades this
Expand Down

0 comments on commit 224e0f8

Please sign in to comment.