aboutsummaryrefslogtreecommitdiffstats
path: root/cparser/Cabs.v
diff options
context:
space:
mode:
authorXavier Leroy <xavier.leroy@college-de-france.fr>2020-07-21 18:42:27 +0200
committerXavier Leroy <xavierleroy@users.noreply.github.com>2020-07-21 18:45:28 +0200
commita8ce85adbf2863e98e5c24e9cc6f82947d4b3a29 (patch)
treec289886f88b58716ecfe0f7261594a231a3b21be /cparser/Cabs.v
parent3a1b0e98a09dd9688e8f45f9677b7ea25f4720bf (diff)
downloadcompcert-kvx-a8ce85adbf2863e98e5c24e9cc6f82947d4b3a29.tar.gz
compcert-kvx-a8ce85adbf2863e98e5c24e9cc6f82947d4b3a29.zip
Support _Static_assert from C11
Diffstat (limited to 'cparser/Cabs.v')
-rw-r--r--cparser/Cabs.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/cparser/Cabs.v b/cparser/Cabs.v
index 5f12e8a1..ff046cba 100644
--- a/cparser/Cabs.v
+++ b/cparser/Cabs.v
@@ -92,6 +92,7 @@ with parameter :=
(* The optional expression is the bitfield *)
with field_group :=
| Field_group : list spec_elem -> list (option name * option expression) -> loc -> field_group
+ | Field_group_static_assert : expression -> loc -> constant -> loc -> loc -> field_group
(* The decl_type is in the order in which they are printed. Only the name of
* the declared identifier is pulled out. *)
@@ -197,6 +198,7 @@ Inductive definition :=
| FUNDEF : list spec_elem -> name -> list definition -> statement -> loc -> definition
| DECDEF : init_name_group -> loc -> definition (* global variable(s), or function prototype *)
| PRAGMA : string -> loc -> definition
+ | STATIC_ASSERT : expression -> loc -> constant -> loc -> loc -> definition
(*
** statements