From 7cc2810b4b1ea92a8f8a8739f69a94d5578e7b9d Mon Sep 17 00:00:00 2001 From: Léo Gourdin Date: Mon, 29 Mar 2021 11:12:07 +0200 Subject: replacing omega with lia in some file --- common/Events.v | 3 ++- 1 file changed, 2 insertions(+), 1 deletion(-) (limited to 'common/Events.v') diff --git a/common/Events.v b/common/Events.v index 13741ebd..aff9e256 100644 --- a/common/Events.v +++ b/common/Events.v @@ -25,6 +25,7 @@ Require Import Values. Require Import Memory. Require Import Globalenvs. Require Import Builtins. +Require Import Lia. (** * Events and traces *) @@ -1443,7 +1444,7 @@ Proof. econstructor; eauto. red; intros; congruence. (* trace length *) -- inv H; simpl; omega. +- inv H; simpl; lia. (* receptive *) - inv H; inv H0. exists Vundef, m1; constructor. (* determ *) -- cgit