Module Qcert.Compiler.QLib


Require Import CompilerRuntime.
Require QData QOperators.
Require QOQL QSQL QSQLPP QLambdaNRA QCAMP QCAMPRule.
Require QUtil QType QEval.
Require QLang QDriver QStat.

Module QLib(runtime:CompilerRuntime).

  Module QType := QType.QType runtime.
  Module QData := QData.QData runtime.
  Module QOps := QOperators.QOperators runtime.

  Module QOQL := QOQL.QOQL runtime.
  Module QSQL := QSQL.QSQL runtime.
  Module QSQLPP := QSQLPP.QSQLPP runtime.
  Module QLambdaNRA := QLambdaNRA.QLambdaNRA runtime.
  Module QCAMP := QCAMP.QCAMP runtime.
  Module QCAMPRule := QCAMPRule.QCAMPRule runtime.

  Module QLang := QLang.QLang runtime.
  Module QDriver := QDriver.QDriver runtime.
  Module QStat := QStat.QStat runtime.
  Module QUtil := QUtil.QUtil runtime.

  Module QEval := QEval.QEval runtime.

End QLib.