aboutsummaryrefslogtreecommitdiffstats
path: root/kvx/Asmvliw.v
diff options
context:
space:
mode:
Diffstat (limited to 'kvx/Asmvliw.v')
-rw-r--r--kvx/Asmvliw.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/kvx/Asmvliw.v b/kvx/Asmvliw.v
index 8afe8d07..aa2e0885 100644
--- a/kvx/Asmvliw.v
+++ b/kvx/Asmvliw.v
@@ -32,6 +32,7 @@ Require Import Conventions.
Require Import Errors.
Require Import Sorting.Permutation.
Require Import Chunks.
+Require Import Lia.
(** * Abstract syntax *)
@@ -1709,7 +1710,7 @@ Ltac Det_WIO X :=
split. auto. intros. destruct B; auto. subst. auto.
- (* trace length *)
red; intros. inv H; cbn.
- omega.
+ lia.
eapply external_call_trace_length; eauto.
eapply external_call_trace_length; eauto.
- (* initial states *)