aboutsummaryrefslogtreecommitdiff
path: root/theories/FSets
diff options
context:
space:
mode:
authorPierre-Marie Pédrot2018-09-11 11:46:10 +0200
committerPierre-Marie Pédrot2018-09-11 11:46:10 +0200
commit2f0e274a1436b477e0be0be94a36ee9461a89767 (patch)
tree536189bce5ef6f21565fb32534bae11cc37ead2a /theories/FSets
parentf3475cd1a68f632b1e6522975354c7dcc1acd6bb (diff)
parentddc25ec6150005e949442d422549fbc213d8f4af (diff)
Merge PR #8425: Deprecate romega in favor of lia
Diffstat (limited to 'theories/FSets')
-rw-r--r--theories/FSets/FMapFullAVL.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/FSets/FMapFullAVL.v b/theories/FSets/FMapFullAVL.v
index 3452967821..c0db8646c7 100644
--- a/theories/FSets/FMapFullAVL.v
+++ b/theories/FSets/FMapFullAVL.v
@@ -27,7 +27,7 @@
*)
-Require Import FunInd Recdef FMapInterface FMapList ZArith Int FMapAVL ROmega.
+Require Import FunInd Recdef FMapInterface FMapList ZArith Int FMapAVL Lia.
Set Implicit Arguments.
Unset Strict Implicit.
@@ -39,7 +39,7 @@ Import Raw.Proofs.
Local Open Scope pair_scope.
Local Open Scope Int_scope.
-Ltac omega_max := i2z_refl; romega with Z.
+Ltac omega_max := i2z_refl; lia.
Section Elt.
Variable elt : Type.
@@ -697,7 +697,7 @@ Module IntMake_ord (I:Int)(X: OrderedType)(D : OrderedType) <:
end.
Proof.
intros; unfold cardinal_e_2; simpl;
- abstract (do 2 rewrite cons_cardinal_e; romega with * ).
+ abstract (do 2 rewrite cons_cardinal_e; lia ).
Defined.
Definition Cmp c :=