aboutsummaryrefslogtreecommitdiffstats
path: root/backend/LTLtyping.v
diff options
context:
space:
mode:
Diffstat (limited to 'backend/LTLtyping.v')
-rw-r--r--backend/LTLtyping.v6
1 files changed, 6 insertions, 0 deletions
diff --git a/backend/LTLtyping.v b/backend/LTLtyping.v
index 0461c9af..e62f9287 100644
--- a/backend/LTLtyping.v
+++ b/backend/LTLtyping.v
@@ -94,6 +94,12 @@ Inductive wt_instr : instruction -> Prop :=
locs_acceptable args ->
valid_successor s1 -> valid_successor s2 ->
wt_instr (Lcond cond args s1 s2)
+ | wt_Ljumptable:
+ forall arg tbl,
+ Loc.type arg = Tint ->
+ loc_acceptable arg ->
+ (forall lbl, In lbl tbl -> valid_successor lbl) ->
+ wt_instr (Ljumptable arg tbl)
| wt_Lreturn:
forall optres,
option_map Loc.type optres = funct.(fn_sig).(sig_res) ->