Theory CoCallImplTTree

theory CoCallImplTTree
imports TTreeAnalysisSig "Env-Set-Cpo" CoCallAritySig "CoCallGraph-TTree"
begin

context CoCallArity
begin
  definition Texp :: "exp  Arity  var ttree"
    where "Texp e = (Λ a. ccTTree (edom (Aexp e a)) (ccExp ea))"
  
  lemma Texp_simp: "Texp ea = ccTTree (edom (Aexp e a)) (ccExp ea)"
    unfolding Texp_def
    by simp

  sublocale TTreeAnalysis Texp.
end



end