renamed "emb" to "list_hembeq";
make "list_hembeq" reflexive independent of the base order;
renamed "sub" to "sublisteq";
dropped "transp_on" (state transitivity explicitly instead);
no need to hide "sub" after renaming;
replaced some ASCII symbols by proper Isabelle symbols;
NEWS
(* Title: HOL/Library/Quotient_Syntax.thy
Author: Cezary Kaliszyk and Christian Urban
*)
header {* Pretty syntax for Quotient operations *}
theory Quotient_Syntax
imports Main
begin
notation
rel_conj (infixr "OOO" 75) and
map_fun (infixr "--->" 55) and
fun_rel (infixr "===>" 55)
end