-
Notifications
You must be signed in to change notification settings - Fork 0
/
Copy pathExtraction_Haskell_String_12258.v
52 lines (47 loc) · 1.82 KB
/
Extraction_Haskell_String_12258.v
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
39
40
41
42
43
44
45
46
47
48
49
50
51
52
Require Import Stdlib.extraction.Extraction.
Require Import Stdlib.extraction.ExtrHaskellString.
Extraction Language Haskell.
Set Extraction File Comment "IMPORTANT: If you change this file, make sure that running [cp Extraction_Haskell_String_12258.out Extraction_Haskell_String_12258.hs && ghc -o test Extraction_Haskell_String_12258.hs] succeeds".
Inductive output_type_code :=
| ascii_dec
| ascii_eqb
| string_dec
| string_eqb
| byte_eqb
| byte_eq_dec
.
Definition output_type_sig (c : output_type_code) : { T : Type & T }
:= existT (fun T => T)
_
match c return match c with ascii_dec => _ | _ => _ end with
| ascii_dec => Ascii.ascii_dec
| ascii_eqb => Ascii.eqb
| string_dec => String.string_dec
| string_eqb => String.eqb
| byte_eqb => Byte.eqb
| byte_eq_dec => Byte.byte_eq_dec
end.
Definition output_type (c : output_type_code)
:= Eval cbv [output_type_sig projT1 projT2] in
projT1 (output_type_sig c).
Definition output (c : output_type_code) : output_type c
:= Eval cbv [output_type_sig projT1 projT2] in
match c return output_type c with
| ascii_dec as c
| _ as c
=> projT2 (output_type_sig c)
end.
Axiom IO_unit : Set.
Axiom _IO : Set -> Set.
Axiom _IO_bind : forall {A B}, _IO A -> (A -> _IO B) -> _IO B.
Axiom _IO_return : forall {A : Set}, A -> _IO A.
Axiom cast_io : _IO unit -> IO_unit.
Extract Constant _IO "a" => "GHC.Base.IO a".
Extract Inlined Constant _IO_bind => "(Prelude.>>=)".
Extract Inlined Constant _IO_return => "GHC.Base.return".
Extract Inlined Constant IO_unit => "GHC.Base.IO ()".
Extract Inlined Constant cast_io => "".
Definition main : IO_unit
:= cast_io (_IO_bind (_IO_return output)
(fun _ => _IO_return tt)).
Recursive Extraction main.