aboutsummaryrefslogtreecommitdiffstats
path: root/flocq/Calc/Operations.v
diff options
context:
space:
mode:
authorGuillaume Melquiond <guillaume.melquiond@inria.fr>2020-12-28 15:53:36 +0100
committerGitHub <noreply@github.com>2020-12-28 15:53:36 +0100
commitd4513f41c54869c9b4ba96ab79d50933a1d5c25a (patch)
treeb5ef5b74c19f386791d1f572c45b6b7af0e90451 /flocq/Calc/Operations.v
parent548e62be073aa5a7b39d5826cd72681daef7c6a1 (diff)
downloadcompcert-kvx-d4513f41c54869c9b4ba96ab79d50933a1d5c25a.tar.gz
compcert-kvx-d4513f41c54869c9b4ba96ab79d50933a1d5c25a.zip
Update Flocq to 3.4.0 (#383)
Diffstat (limited to 'flocq/Calc/Operations.v')
-rw-r--r--flocq/Calc/Operations.v6
1 files changed, 4 insertions, 2 deletions
diff --git a/flocq/Calc/Operations.v b/flocq/Calc/Operations.v
index 3416cb4e..ac93d412 100644
--- a/flocq/Calc/Operations.v
+++ b/flocq/Calc/Operations.v
@@ -17,7 +17,9 @@ MERCHANTABILITY or FITNESS FOR A PARTICULAR PURPOSE. See the
COPYING file for more details.
*)
-(** Basic operations on floats: alignment, addition, multiplication *)
+(** * Basic operations on floats: alignment, addition, multiplication *)
+
+From Coq Require Import Lia.
Require Import Raux Defs Float_prop.
Set Implicit Arguments.
@@ -50,7 +52,7 @@ case (Zle_bool e1 e2) ; intros He ; split ; trivial.
now rewrite <- F2R_change_exp.
rewrite <- F2R_change_exp.
apply refl_equal.
-omega.
+lia.
Qed.
Theorem Falign_spec_exp: