Module Qcert.Translation.Operators.ForeignToScala


Require Import List.
Require Import String.
Require Import Utils.
Require Import ForeignRuntime.
Require Import ForeignType.

Local Open Scope string_scope.

Section ForeigntoScala.

  Class foreign_to_scala {fruntime:foreign_runtime} {ftype: foreign_type}: Type
    := mk_foreign_to_scala {
           foreign_to_scala_unary_op
             (fu:foreign_operators_unary)
             (d:string) : string
           ; foreign_to_scala_spark_datatype (ft: foreign_type_type) : string
         }.

End ForeigntoScala.