aboutsummaryrefslogtreecommitdiffstats
path: root/lib/IEEE754_extra.v
diff options
context:
space:
mode:
authorXavier Leroy <xavier.leroy@college-de-france.fr>2020-09-21 14:15:57 +0200
committerXavier Leroy <xavier.leroy@college-de-france.fr>2020-09-21 14:37:38 +0200
commitab0d9476db875a82cf293623d18552b62f239d5c (patch)
treec6c121933c1b536f03f5b8386f8b351c315763d8 /lib/IEEE754_extra.v
parentb525fbe0915931a939d5851b511ce46fcf026236 (diff)
downloadcompcert-kvx-ab0d9476db875a82cf293623d18552b62f239d5c.tar.gz
compcert-kvx-ab0d9476db875a82cf293623d18552b62f239d5c.zip
Support the use of already-installed MenhirLib and Flocq libraries
configure flags -use-external-Flocq and -use external-MenhirLib.
Diffstat (limited to 'lib/IEEE754_extra.v')
-rw-r--r--lib/IEEE754_extra.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/lib/IEEE754_extra.v b/lib/IEEE754_extra.v
index c23149be..18313ec1 100644
--- a/lib/IEEE754_extra.v
+++ b/lib/IEEE754_extra.v
@@ -17,11 +17,11 @@
(** Additional operations and proofs about IEEE-754 binary
floating-point numbers, on top of the Flocq library. *)
+From Flocq Require Import Core Digits Operations Round Bracket Sterbenz
+ Binary Round_odd.
Require Import Psatz.
Require Import Bool.
Require Import Eqdep_dec.
-(*From Flocq *)
-Require Import Core Digits Operations Round Bracket Sterbenz Binary Round_odd.
Local Open Scope Z_scope.