Quot/Quotient_Syntax.thy
changeset 1130 fb5f5735a426
child 1148 389d81959922
equal deleted inserted replaced
1129:9a86f0ef6503 1130:fb5f5735a426
       
     1 header {* Pretty syntax for Quotient operations *}
       
     2 
       
     3 (*<*)
       
     4 theory Quotient_Syntax
       
     5 imports Quotient
       
     6 begin
       
     7 
       
     8 notation
       
     9   rel_conj (infixr "OOO" 75) and
       
    10   fun_map (infixr "--->" 55) and
       
    11   fun_rel (infixr "===>" 55)
       
    12 
       
    13 end
       
    14 (*>*)