Skip to content

Commit

Permalink
chore: remove ported tactic from Mathport syntax (#14385)
Browse files Browse the repository at this point in the history
`move_add`, `move_mul` and `move_oper` are all available in `Mathlib`.
  • Loading branch information
adomani committed Jul 3, 2024
1 parent e6737c3 commit 343699a
Showing 1 changed file with 0 additions and 6 deletions.
6 changes: 0 additions & 6 deletions Mathlib/Mathport/Syntax.lean
Original file line number Diff line number Diff line change
Expand Up @@ -253,12 +253,6 @@ syntax generalizingClause := " generalizing" (ppSpace ident)+

/- E -/ syntax (name := wittTruncateFunTac) "witt_truncate_fun_tac" : tactic

/- M -/ syntax (name := moveOp) "move_op " term:max ppSpace rwRule,+ (location)? : tactic
macro (name := moveMul) "move_mul " pats:rwRule,+ loc:(location)? : tactic =>
`(tactic| move_op (·*·) $pats,* $(loc)?)
macro (name := moveAdd) "move_add " pats:rwRule,+ loc:(location)? : tactic =>
`(tactic| move_op (·+·) $pats,* $(loc)?)

/- S -/ syntax (name := intro) "intro" : attr
/- S -/ syntax (name := intro!) "intro!" : attr

Expand Down

0 comments on commit 343699a

Please sign in to comment.