aboutsummaryrefslogtreecommitdiff
path: root/plugins/extraction/ExtrHaskellNatInt.v
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2020-02-05 17:46:07 +0100
committerEmilio Jesus Gallego Arias2020-02-13 21:12:03 +0100
commit9193769161e1f06b371eed99dfe9e90fec9a14a6 (patch)
treee16e5f60ce6a88656ccd802d232cde6171be927d /plugins/extraction/ExtrHaskellNatInt.v
parenteb83c142eb33de18e3bfdd7c32ecfb797a640c38 (diff)
[build] Consolidate stdlib's .v files under a single directory.
Currently, `.v` under the `Coq.` prefix are found in both `theories` and `plugins`. Usually these two directories are merged by special loadpath code that allows double-binding of the prefix. This adds some complexity to the build and loadpath system; and in particular, it prevents from handling the `Coq.*` prefix in the simple, `-R theories Coq` standard way. We thus move all `.v` files to theories, leaving `plugins` as an OCaml-only directory, and modify accordingly the loadpath / build infrastructure. Note that in general `plugins/foo/Foo.v` was not self-contained, in the sense that it depended on files in `theories` and files in `theories` depended on it; moreover, Coq saw all these files as belonging to the same namespace so it didn't really care where they lived. This could also imply a performance gain as we now effectively traverse less directories when locating a library. See also discussion in #10003
Diffstat (limited to 'plugins/extraction/ExtrHaskellNatInt.v')
-rw-r--r--plugins/extraction/ExtrHaskellNatInt.v15
1 files changed, 0 insertions, 15 deletions
diff --git a/plugins/extraction/ExtrHaskellNatInt.v b/plugins/extraction/ExtrHaskellNatInt.v
deleted file mode 100644
index 267322d9ed..0000000000
--- a/plugins/extraction/ExtrHaskellNatInt.v
+++ /dev/null
@@ -1,15 +0,0 @@
-(** Extraction of [nat] into Haskell's [Int] *)
-
-Require Coq.extraction.Extraction.
-
-Require Import Arith.
-Require Import ExtrHaskellNatNum.
-
-(**
- * Disclaimer: trying to obtain efficient certified programs
- * by extracting [nat] into [Int] is definitively *not* a good idea.
- * See comments in [ExtrOcamlNatInt.v].
- *)
-
-Extract Inductive nat => "Prelude.Int" [ "0" "Prelude.succ" ]
- "(\fO fS n -> if n Prelude.== 0 then fO () else fS (n Prelude.- 1))".