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 --- kvx/Asmblockgenproof.v | 15 ++++++++------- 1 file changed, 8 insertions(+), 7 deletions(-) (limited to 'kvx/Asmblockgenproof.v') diff --git a/kvx/Asmblockgenproof.v b/kvx/Asmblockgenproof.v index df1a070f..6e3029d8 100644 --- a/kvx/Asmblockgenproof.v +++ b/kvx/Asmblockgenproof.v @@ -21,6 +21,7 @@ Require Import Values Memory Events Globalenvs Smallstep. Require Import Op Locations Machblock Conventions Asmblock. Require Import Asmblockgen Asmblockgenproof0 Asmblockgenproof1 Asmblockprops. Require Import Axioms. +Require Import Lia. Module MB := Machblock. Module AB := Asmvliw. @@ -72,7 +73,7 @@ Lemma transf_function_no_overflow: transf_function f = OK tf -> size_blocks tf.(fn_blocks) <= Ptrofs.max_unsigned. Proof. intros. monadInv H. destruct (zlt Ptrofs.max_unsigned (size_blocks x.(fn_blocks))); inv EQ0. - omega. + lia. Qed. Section TRANSL_LABEL. (* Lemmas on translation of MB.is_label into AB.is_label *) @@ -247,8 +248,8 @@ Proof. split. unfold goto_label. unfold par_goto_label. rewrite P. rewrite H1. auto. split. rewrite Pregmap.gss. constructor; auto. rewrite Ptrofs.unsigned_repr. replace (pos' - 0) with pos' in Q. - auto. omega. - generalize (transf_function_no_overflow _ _ H0). omega. + auto. lia. + generalize (transf_function_no_overflow _ _ H0). lia. intros. apply Pregmap.gso; auto. Qed. @@ -1374,7 +1375,7 @@ Lemma mbsize_eqz: Proof. intros. destruct bb as [hd bdy ex]; simpl in *. unfold mbsize in H. remember (length _) as a. remember (length_opt _) as b. - assert (a = 0%nat) by omega. assert (b = 0%nat) by omega. subst. clear H. + assert (a = 0%nat) by lia. assert (b = 0%nat) by lia. subst. clear H. inv H0. inv H1. destruct bdy; destruct ex; auto. all: try discriminate. Qed. @@ -1706,11 +1707,11 @@ Proof. + contradiction. } destruct EXEC_PROLOGUE as (rs3' & EXEC_PROLOGUE & Heqrs3'). exploit exec_straight_steps_2; eauto using functions_transl. - simpl fn_blocks. simpl fn_blocks in g. omega. constructor. + simpl fn_blocks. simpl fn_blocks in g. lia. constructor. intros (ofs' & X & Y). left; exists (State rs3' m3'); split. eapply exec_straight_steps_1; eauto. - simpl fn_blocks. simpl fn_blocks in g. omega. + simpl fn_blocks. simpl fn_blocks in g. lia. constructor. econstructor; eauto. rewrite X; econstructor; eauto. @@ -1756,7 +1757,7 @@ Local Transparent destroyed_at_function_entry. - (* return *) inv MS. inv STACKS. simpl in *. - right. split. omega. split. auto. + right. split. lia. split. auto. rewrite <- ATPC in H5. econstructor; eauto. congruence. Qed. -- cgit