diff options
| author | Maxime Dénès | 2020-01-08 14:42:33 +0100 |
|---|---|---|
| committer | Maxime Dénès | 2020-01-08 15:07:29 +0100 |
| commit | 3e89f884ef60eb54b250632bb55131e7258ae813 (patch) | |
| tree | e5d4b6485ce872e6ddcfe37460e633f3dc95b26b /test-suite/output/ExtractionString.v | |
| parent | ef938a4ce2c03b1c4f23222a4542ad144a1f209b (diff) | |
Add test case for string extraction in OCaml and Haskell
Diffstat (limited to 'test-suite/output/ExtractionString.v')
| -rw-r--r-- | test-suite/output/ExtractionString.v | 25 |
1 files changed, 25 insertions, 0 deletions
diff --git a/test-suite/output/ExtractionString.v b/test-suite/output/ExtractionString.v new file mode 100644 index 0000000000..e4b9d22b38 --- /dev/null +++ b/test-suite/output/ExtractionString.v @@ -0,0 +1,25 @@ +Require Import String Extraction. + +Definition str := "This is a string"%string. + +(* Raw extraction of strings, in OCaml *) +Extraction Language OCaml. +Extraction str. + +(* Raw extraction of strings, in Haskell *) +Extraction Language Haskell. +Extraction str. + +(* Extraction to char list, in OCaml *) +Require Import ExtrOcamlString. +Extraction Language OCaml. +Extraction str. + +(* Extraction to native strings, in OCaml *) +Require Import ExtrOcamlNativeString. +Extraction str. + +(* Extraction to native strings, in Haskell *) +Require Import ExtrHaskellString. +Extraction Language Haskell. +Extraction str. |
