Library Io.System.Extraction
Extraction to OCaml. New primitives are defined in `extraction/utils.ml`. 
Require Import Coq.Lists.List.
Require Import Coq.PArith.PArith.
Require Import Coq.ZArith.ZArith.
Require Import ExtrOcamlBasic.
Require Import ExtrOcamlString.
Require Import ErrorHandlers.All.
Require Import FunctionNinjas.All.
Require Import ListString.All.
Require Import Io.All.
Require System.
Import ListNotations.
Local Open Scope type.
Require Import Coq.PArith.PArith.
Require Import Coq.ZArith.ZArith.
Require Import ExtrOcamlBasic.
Require Import ExtrOcamlString.
Require Import ErrorHandlers.All.
Require Import FunctionNinjas.All.
Require Import ListString.All.
Require Import Io.All.
Require System.
Import ListNotations.
Local Open Scope type.
Interface to the Big_int library. 
The OCaml's `big_int` type. 
  Parameter t : Type.
Extract Constant t ⇒ "Big_int.big_int".
Parameter to_Z_aux : ∀ {Z positive : Type},
t →
Z → (positive → Z) → (positive → Z) →
positive → (positive → positive) → (positive → positive) →
Z.
Extract Constant to_Z_aux ⇒ "IoSystem.Big.to_Z_aux".
Extract Constant t ⇒ "Big_int.big_int".
Parameter to_Z_aux : ∀ {Z positive : Type},
t →
Z → (positive → Z) → (positive → Z) →
positive → (positive → positive) → (positive → positive) →
Z.
Extract Constant to_Z_aux ⇒ "IoSystem.Big.to_Z_aux".
Export to a `Z`. 
Interface with the OCaml strings. 
The OCaml `string` type. 
Export to an OCaml string. 
Import an OCaml string. 
  Parameter to_lstring : t → LString.t.
Extract Constant to_lstring ⇒ "IoSystem.String.to_lstring".
End String.
Extract Constant to_lstring ⇒ "IoSystem.String.to_lstring".
End String.
Interface to the Sys library. 
The command line arguments of the program. 
Interface to the Lwt library. 
The `Lwt.t` type. 
Return. 
Bind. 
Join. 
Choose. 
Launch. 
List the files of a directory. 
  Parameter list_files : String.t → t (option (list String.t)).
Extract Constant list_files ⇒ "IoSystem.list_files".
Extract Constant list_files ⇒ "IoSystem.list_files".
The the content of a file. 
  Parameter read_file : String.t → t (option String.t).
Extract Constant read_file ⇒ "IoSystem.read_file".
Extract Constant read_file ⇒ "IoSystem.read_file".
Update (or create) a file with some content. 
  Parameter write_file : String.t → String.t → t bool.
Extract Constant write_file ⇒ "IoSystem.write_file".
Extract Constant write_file ⇒ "IoSystem.write_file".
Delete a file. 
Run a command. 
Run a command controlling the outputs. 
  Parameter eval : list String.t → t (option (BigInt.t × String.t × String.t)).
Extract Constant eval ⇒ "IoSystem.eval".
Extract Constant eval ⇒ "IoSystem.eval".
Print a message on the standard output. 
Read a line on the standard input. 
  Parameter read_line : unit → t (option String.t).
Extract Constant read_line ⇒ "IoSystem.read_line".
End Lwt.
Extract Constant read_line ⇒ "IoSystem.read_line".
End Lwt.
Evaluate a command using Lwt. 
Definition eval_command (c : Effect.command System.effect)
: Lwt.t (Effect.answer System.effect c) :=
match c return (Lwt.t (Effect.answer System.effect c)) with
| System.ListFiles folder ⇒
Lwt.bind (Lwt.list_files @@ String.of_lstring folder) (fun files ⇒
Lwt.ret @@ Option.bind files (fun files ⇒
Some (List.map String.to_lstring files)))
| System.ReadFile file_name ⇒
Lwt.bind (Lwt.read_file @@ String.of_lstring file_name) (fun content ⇒
Lwt.ret @@ option_map String.to_lstring content)
| System.WriteFile file_name content ⇒
let file_name := String.of_lstring file_name in
let content := String.of_lstring content in
Lwt.write_file file_name content
| System.DeleteFile file_name ⇒
Lwt.delete_file @@ String.of_lstring file_name
| System.System command ⇒ Lwt.system (String.of_lstring command)
| System.Eval command ⇒
let command := List.map String.of_lstring command in
Lwt.bind (Lwt.eval command) (fun result ⇒
Lwt.ret (result |> option_map (fun result ⇒
match result with
| (status, output, err) ⇒
(BigInt.to_Z status, String.to_lstring output, String.to_lstring err)
end)))
| System.Print message ⇒
let message := String.of_lstring message in
Lwt.print message
| System.ReadLine ⇒
Lwt.bind (Lwt.read_line tt) (fun line ⇒
Lwt.ret @@ option_map String.to_lstring line)
end.
: Lwt.t (Effect.answer System.effect c) :=
match c return (Lwt.t (Effect.answer System.effect c)) with
| System.ListFiles folder ⇒
Lwt.bind (Lwt.list_files @@ String.of_lstring folder) (fun files ⇒
Lwt.ret @@ Option.bind files (fun files ⇒
Some (List.map String.to_lstring files)))
| System.ReadFile file_name ⇒
Lwt.bind (Lwt.read_file @@ String.of_lstring file_name) (fun content ⇒
Lwt.ret @@ option_map String.to_lstring content)
| System.WriteFile file_name content ⇒
let file_name := String.of_lstring file_name in
let content := String.of_lstring content in
Lwt.write_file file_name content
| System.DeleteFile file_name ⇒
Lwt.delete_file @@ String.of_lstring file_name
| System.System command ⇒ Lwt.system (String.of_lstring command)
| System.Eval command ⇒
let command := List.map String.of_lstring command in
Lwt.bind (Lwt.eval command) (fun result ⇒
Lwt.ret (result |> option_map (fun result ⇒
match result with
| (status, output, err) ⇒
(BigInt.to_Z status, String.to_lstring output, String.to_lstring err)
end)))
| System.Print message ⇒
let message := String.of_lstring message in
Lwt.print message
| System.ReadLine ⇒
Lwt.bind (Lwt.read_line tt) (fun line ⇒
Lwt.ret @@ option_map String.to_lstring line)
end.
Evaluate an expression using Lwt. 
Fixpoint eval {A : Type} (x : C.t System.effect A) : Lwt.t A.
destruct x as [A x | command | A B x f | A x1 x2 | A B x y].
- exact (Lwt.ret x).
- exact (eval_command command).
- exact (Lwt.bind (eval _ x) (fun x ⇒ eval _ (f x))).
- exact (Lwt.choose (eval _ x1) (eval _ x2)).
- exact (Lwt.join (eval _ x) (eval _ y)).
Defined.
destruct x as [A x | command | A B x f | A x1 x2 | A B x y].
- exact (Lwt.ret x).
- exact (eval_command command).
- exact (Lwt.bind (eval _ x) (fun x ⇒ eval _ (f x))).
- exact (Lwt.choose (eval _ x1) (eval _ x2)).
- exact (Lwt.join (eval _ x) (eval _ y)).
Defined.
Launch the main function. 
Definition launch (main : list LString.t → C.t System.effect unit) : unit :=
let argv := List.map String.to_lstring Sys.argv in
Lwt.launch (eval (main argv)).
let argv := List.map String.to_lstring Sys.argv in
Lwt.launch (eval (main argv)).