aboutsummaryrefslogtreecommitdiffstats
path: root/MenhirLib/Automaton.v
diff options
context:
space:
mode:
authorJacques-Henri Jourdan <jacques-henri.jourdan@normalesup.org>2019-07-06 16:16:20 +0200
committerXavier Leroy <xavierleroy@users.noreply.github.com>2019-07-06 16:16:20 +0200
commit415c5a5a28ac7035cfa33e5753af841a450bfab0 (patch)
treeef38884d5d3a2a4207d481b32ac7d898859bb04d /MenhirLib/Automaton.v
parent5e8cac37b13cd3dcfbbe8e9dd939ed1fa9d5e310 (diff)
downloadcompcert-kvx-415c5a5a28ac7035cfa33e5753af841a450bfab0.tar.gz
compcert-kvx-415c5a5a28ac7035cfa33e5753af841a450bfab0.zip
Fix compatibility with Coq 8.10 (#303)
The generation of some fresh names changes in Coq 8.10 (https://github.com/coq/coq/pull/9160). The `Hint Mode` declaration that does not specify a hint database now triggers a warning. Specify the intended database and fix the "auto" tactics accordingly.
Diffstat (limited to 'MenhirLib/Automaton.v')
-rw-r--r--MenhirLib/Automaton.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/MenhirLib/Automaton.v b/MenhirLib/Automaton.v
index c310fc61..d5a19f35 100644
--- a/MenhirLib/Automaton.v
+++ b/MenhirLib/Automaton.v
@@ -99,9 +99,9 @@ Module Types(Import Init:AutInit).
T term = last_symb_of_non_init_state s -> lookahead_action term
| Reduce_act: production -> lookahead_action term
| Fail_act: lookahead_action term.
- Arguments Shift_act [term].
- Arguments Reduce_act [term].
- Arguments Fail_act [term].
+ Arguments Shift_act {term}.
+ Arguments Reduce_act {term}.
+ Arguments Fail_act {term}.
Inductive action :=
| Default_reduce_act: production -> action