Theory CoCallAnalysisSig

theory CoCallAnalysisSig
imports Launchbury.Terms Arity CoCallGraph
begin

locale CoCallAnalysis =
  fixes ccExp :: "exp  Arity  CoCalls"
begin
  abbreviation ccExp_syn ("𝒢⇘_")
    where "𝒢⇘a (λe. ccExp ea)"
  abbreviation ccExp_bot_syn ("𝒢_")
    where "𝒢a (λe. fup(ccExp e)a)"
end

locale CoCallAnalyisHeap = 
  fixes ccHeap :: "heap  exp  Arity  CoCalls"

end