Module Qcert.TechRule.Lang.TechRule


TechRule stands for ODM technical rules. This is merely a place-holder since the source language is effectively parsed in Java.

Summary:

Require Import Utils.
Require Import DataRuntime.
Require Export CAMPRuleRuntime.

Section TechRule.
  Context {fruntime:foreign_runtime}.

  Axiom tech_rule : Set.
  Axiom tech_rule_to_camp_rule : tech_rule -> camp_rule.

End TechRule.