aboutsummaryrefslogtreecommitdiffstats
path: root/backend/Debugvar.v
diff options
context:
space:
mode:
authorXavier Leroy <xavier.leroy@college-de-france.fr>2020-06-21 19:14:32 +0200
committerXavier Leroy <xavier.leroy@college-de-france.fr>2020-06-21 19:14:32 +0200
commit70609c932e066ffab0d2e3a2a38d66e834399532 (patch)
tree1a70c96a611508a98c6f967bf5eabdd06ae4f6f3 /backend/Debugvar.v
parent375c844efb8b91d4ff1dce08ed25f55ddef231d7 (diff)
downloadcompcert-kvx-70609c932e066ffab0d2e3a2a38d66e834399532.tar.gz
compcert-kvx-70609c932e066ffab0d2e3a2a38d66e834399532.zip
Transform non-recursive Fixpoint into Definition
As detected by the new warning in Coq 8.12. The use of Fixpoint here is not warranted and either an oversight or a leftover from an earlier version.
Diffstat (limited to 'backend/Debugvar.v')
-rw-r--r--backend/Debugvar.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/backend/Debugvar.v b/backend/Debugvar.v
index 1f361030..3204dae5 100644
--- a/backend/Debugvar.v
+++ b/backend/Debugvar.v
@@ -92,7 +92,7 @@ Fixpoint remove_state (v: ident) (s: avail) : avail :=
end
end.
-Fixpoint set_debug_info (v: ident) (info: list (builtin_arg loc)) (s: avail) :=
+Definition set_debug_info (v: ident) (info: list (builtin_arg loc)) (s: avail) :=
match normalize_debug info with
| Some a => set_state v a s
| None => remove_state v s