Module Qcert.Translation.Lang.TechRuletoCAMPRule


Require Import String.
Require Import List.
Require Import DataRuntime.
Require Import TechRuleRuntime.
Require Import CAMPRuleRuntime.
  
Section TechRuletoCAMPRule.
  Section Top.
    Context {fr:foreign_runtime}.

Note: Translation from Tech Rules to CAMP Rule is done in Java
    Definition tech_rule_to_camp_rule_top (q:tech_rule) : camp_rule :=
      tech_rule_to_camp_rule q.
  End Top.
    
End TechRuletoCAMPRule.