Theory First_Order_Clause.Tiebreakers

theory Tiebreakers
  imports Restricted_Order Nonground_Clause_Generic
begin

type_synonym ('g, 'a) tiebreakers = 
  "'g clause  'a clause  'a clause  bool"

locale tiebreakers =
  fixes tiebreakers :: "('g, 'a) tiebreakers"
  assumes "CG. wfp (tiebreakers CG)  transp (tiebreakers CG)"
begin

sublocale wellfounded_strict_order "tiebreakers CG"
  using tiebreakers_axioms tiebreakers_def wfp_imp_asymp
  by unfold_locales auto  

end

end