Module TechRuletoCAMPRule


Section TechRuletoCAMPRule.
  Require Import String.
  Require Import List.
  Require Import BasicRuntime.
  Require Import TechRuleRuntime.
  Require Import CAMPRuleRuntime.
  
  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.