Skip to content

Commit

Permalink
Fully removing binder_tactic.
Browse files Browse the repository at this point in the history
  • Loading branch information
herbelin committed Dec 6, 2023
1 parent 3c1cf6c commit 2bd0e5b
Show file tree
Hide file tree
Showing 7 changed files with 3 additions and 17 deletions.
4 changes: 2 additions & 2 deletions doc/tools/docgram/README.md
Original file line number Diff line number Diff line change
Expand Up @@ -44,15 +44,15 @@ for documentation purposes:
```
ltac_expr:
[ "5" RIGHTA
[ te = binder_tactic -> { te } ]
[ ... ]
[ "4" ...
```
becomes
```
tactic_expr5: [
| binder_tactic
| ...
| tactic_expr4
]
```
Expand Down
3 changes: 0 additions & 3 deletions doc/tools/docgram/fullGrammar
Original file line number Diff line number Diff line change
Expand Up @@ -2100,9 +2100,6 @@ failkw: [
| "gfail"
]

binder_tactic: [
]

tactic_arg: [
| tactic_value
| Constr.constr
Expand Down
3 changes: 0 additions & 3 deletions doc/tools/docgram/orderedGrammar
Original file line number Diff line number Diff line change
Expand Up @@ -2226,9 +2226,6 @@ ltac_expr0: [
| tactic_atom
]

binder_tactic: [
]

tactic_atom: [
| integer
| qualid
Expand Down
7 changes: 1 addition & 6 deletions plugins/ltac/g_ltac.mlg
Original file line number Diff line number Diff line change
Expand Up @@ -70,7 +70,7 @@ let for_extraargs = ()
}

GRAMMAR EXTEND Gram
GLOBAL: tactic tacdef_body ltac_expr binder_tactic tactic_value command hint
GLOBAL: tactic tacdef_body ltac_expr tactic_value command hint
tactic_mode constr_may_eval constr_eval toplevel_selector
term;

Expand Down Expand Up @@ -164,11 +164,6 @@ GRAMMAR EXTEND Gram
failkw:
[ [ IDENT "fail" -> { TacLocal } | IDENT "gfail" -> { TacGlobal } ] ]
;
(* binder_tactic: level 1 of ltac_expr *)
binder_tactic:
[ RIGHTA
[ ] ]
;
(* Tactic arguments to the right of an application *)
tactic_arg:
[ [ a = tactic_value -> { a }
Expand Down
1 change: 0 additions & 1 deletion plugins/ltac/pltac.ml
Original file line number Diff line number Diff line change
Expand Up @@ -40,7 +40,6 @@ let clause_dft_concl =
(* Main entries for ltac *)
let tactic_value = Entry.make "tactic_value"
let ltac_expr = Entry.make "ltac_expr"
let binder_tactic = Entry.make "binder_tactic"

let tactic = Entry.make "tactic"

Expand Down
1 change: 0 additions & 1 deletion plugins/ltac/pltac.mli
Original file line number Diff line number Diff line change
Expand Up @@ -34,6 +34,5 @@ val in_clause : Names.lident Locus.clause_expr Entry.t
val clause_dft_concl : Names.lident Locus.clause_expr Entry.t
val tactic_value : raw_tactic_arg Entry.t
val ltac_expr : raw_tactic_expr Entry.t
val binder_tactic : raw_tactic_expr Entry.t
val tactic : raw_tactic_expr Entry.t
val tactic_eoi : raw_tactic_expr Entry.t
1 change: 0 additions & 1 deletion plugins/ltac/tacentries.ml
Original file line number Diff line number Diff line change
Expand Up @@ -620,7 +620,6 @@ let () =
let open Pcoq.Entry in
let entries = [
Any Pltac.ltac_expr;
Any Pltac.binder_tactic;
Any Pltac.simple_tactic;
Any Pltac.tactic_value;
] in
Expand Down

0 comments on commit 2bd0e5b

Please sign in to comment.