Skip to content

Commit

Permalink
Merge PR coq#18035: Document the roughness of the Floats library
Browse files Browse the repository at this point in the history
Reviewed-by: silene
Reviewed-by: JasonGross
Ack-by: jfehrle
Co-authored-by: silene <[email protected]>
  • Loading branch information
coqbot-app[bot] and silene authored Sep 18, 2023
2 parents a99e6ec + 31c3d8b commit b881f18
Show file tree
Hide file tree
Showing 2 changed files with 14 additions and 1 deletion.
9 changes: 9 additions & 0 deletions doc/sphinx/language/coq-library.rst
Original file line number Diff line number Diff line change
Expand Up @@ -989,6 +989,15 @@ Notation Interpretation Precedence Associativity
Floats library
~~~~~~~~~~~~~~

The standard library has a small ``Floats`` module for accessing
processor floating-point operations through the Coq kernel.
However, while this module supports computation and has a bit-level
specification, it doesn't include elaborate theorems, such as a link
to real arithmetic or various error bounds. To do proofs by
reflection, use ``Floats`` in conjunction with the complementary
`Flocq <https://flocq.gitlabpages.inria.fr/>`_ library, which provides
many such theorems.

The library of primitive floating-point arithmetic can be loaded by
requiring module ``Floats``:

Expand Down
6 changes: 5 additions & 1 deletion theories/Floats/Floats.v
Original file line number Diff line number Diff line change
Expand Up @@ -17,7 +17,11 @@
- FloatLemmas: prove a few results involving Z.frexp and Z.ldexp
For a brief overview of the Floats library,
see {{https://coq.inria.fr/distrib/current/refman/language/coq-library.html#floats-library}} *)
see {{https://coq.inria.fr/distrib/current/refman/language/coq-library.html#floats-library}}
N.B.: This library only offers a bit-level specification of floating-point
arithmetic. For a more complete set of theorems, including links with real
arithmetic, see the Flocq library {{https://flocq.gitlabpages.inria.fr/}} *)

Require Export FloatClass.
Require Export PrimFloat.
Expand Down

0 comments on commit b881f18

Please sign in to comment.