Theory TTreeAnalysisSig

theory TTreeAnalysisSig
imports Arity  "TTree-HOLCF"  AnalBinds
begin

locale TTreeAnalysis =
 fixes Texp :: "exp  Arity  var ttree"
begin
  sublocale Texp: ExpAnalysis Texp.
  abbreviation "FBinds == Texp.AnalBinds"
end

end