Theory Term_Order_Notation

theory Term_Order_Notation
  imports Main
begin

locale term_order_notation =
  fixes lesst :: "'t  't  bool"
begin

notation lesst (infix "t" 50)

abbreviation "less_eqt  (≺t)=="

notation less_eqt (infix "t" 50)

end

end