Theory First_Order_Clause.Generic_Context

theory Generic_Context
  imports Context_Notation
begin

locale "context" =
  context_notation +
  assumes
    compose_context_iff [simp]: "(c :: 'c) c' (t :: 't). (c c c')t = cc't" and
    apply_hole [simp]: "t. t = t" and
    apply_context_eq: "c t t'. ct = ct'  t = t'"

end