Skip to content

Commit

Permalink
docs(*): merge rewrite tactic tag into rewriting (#2512)
Browse files Browse the repository at this point in the history
We had two overlapping tags in the docs.



Co-authored-by: Rob Lewis <rob.y.lewis@gmail.com>
  • Loading branch information
robertylewis and robertylewis committed Apr 24, 2020
1 parent 13393e3 commit 00d7da2
Show file tree
Hide file tree
Showing 6 changed files with 7 additions and 7 deletions.
2 changes: 1 addition & 1 deletion src/tactic/converter/apply_congr.lean
Expand Up @@ -94,7 +94,7 @@ add_tactic_doc {
name := "apply_congr",
category := doc_category.tactic,
decl_names := [`conv.interactive.apply_congr],
tags := ["conv", "congruence", "rewrite"]
tags := ["conv", "congruence", "rewriting"]
}

end conv.interactive
2 changes: 1 addition & 1 deletion src/tactic/elide.lean
Expand Up @@ -82,7 +82,7 @@ add_tactic_doc
{ name := "elide / unelide",
category := doc_category.tactic,
decl_names := [`tactic.interactive.elide, `tactic.interactive.unelide],
tags := ["goal management", "context management", "rewrite"] }
tags := ["goal management", "context management", "rewriting"] }

end interactive

Expand Down
2 changes: 1 addition & 1 deletion src/tactic/ext.lean
Expand Up @@ -396,6 +396,6 @@ add_tactic_doc
{ name := "ext1 / ext",
category := doc_category.tactic,
decl_names := [`tactic.interactive.ext1, `tactic.interactive.ext],
tags := ["rewrite", "logic"] }
tags := ["rewriting", "logic"] }

end tactic
2 changes: 1 addition & 1 deletion src/tactic/interactive.lean
Expand Up @@ -42,7 +42,7 @@ add_tactic_doc
{ name := "substs",
category := doc_category.tactic,
decl_names := [`tactic.interactive.substs],
tags := ["rewrite"] }
tags := ["rewriting"] }

/-- Unfold coercion-related definitions -/
meta def unfold_coes (loc : parse location) : tactic unit :=
Expand Down
4 changes: 2 additions & 2 deletions src/tactic/lean_core_docs.lean
Expand Up @@ -576,13 +576,13 @@ add_tactic_doc
{ name := "subst",
category := doc_category.tactic,
decl_names := [`tactic.interactive.subst],
tags := ["core", "rewrite"] }
tags := ["core", "rewriting"] }

add_tactic_doc
{ name := "subst_vars",
category := doc_category.tactic,
decl_names := [`tactic.interactive.subst_vars],
tags := ["core", "rewrite"] }
tags := ["core", "rewriting"] }

add_tactic_doc
{ name := "success_if_fail",
Expand Down
2 changes: 1 addition & 1 deletion src/tactic/rewrite.lean
Expand Up @@ -207,7 +207,7 @@ add_tactic_doc
{ name := "assoc_rewrite",
category := doc_category.tactic,
decl_names := [`tactic.interactive.assoc_rewrite, `tactic.interactive.assoc_rw],
tags := ["rewrite"],
tags := ["rewriting"],
inherit_description_from := `tactic.interactive.assoc_rewrite }

end interactive
Expand Down

0 comments on commit 00d7da2

Please sign in to comment.