aboutsummaryrefslogtreecommitdiffstats
path: root/backend/Stacking.v
diff options
context:
space:
mode:
authorXavier Leroy <xavier.leroy@inria.fr>2015-04-06 11:37:53 +0200
committerXavier Leroy <xavier.leroy@inria.fr>2015-04-06 11:37:53 +0200
commit5dadfeabe2eece08c798f29f0329970b693415cc (patch)
treea3aca241f31e35556b484e7bbe1f5f432dd4e517 /backend/Stacking.v
parent500ef9344e0f80ad0c14806e02130ed26da0704a (diff)
downloadcompcert-kvx-5dadfeabe2eece08c798f29f0329970b693415cc.tar.gz
compcert-kvx-5dadfeabe2eece08c798f29f0329970b693415cc.zip
Harmless typo ('__' instead of '_') causing a warning at extraction time.
Diffstat (limited to 'backend/Stacking.v')
-rw-r--r--backend/Stacking.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/backend/Stacking.v b/backend/Stacking.v
index c17dc038..21cf6b73 100644
--- a/backend/Stacking.v
+++ b/backend/Stacking.v
@@ -135,7 +135,7 @@ Fixpoint transl_annot_arg (fe: frame_env) (a: annot_arg loc) : annot_arg mreg :=
| AA_base (R r) => AA_base r
| AA_base (S Local ofs ty) =>
AA_loadstack (chunk_of_type ty) (Int.repr (offset_of_index fe (FI_local ofs ty)))
- | AA_base (S _ _ __) => AA_int Int.zero (**r never happens *)
+ | AA_base (S _ _ _) => AA_int Int.zero (**r never happens *)
| AA_int n => AA_int n
| AA_long n => AA_long n
| AA_float n => AA_float n