Attic/Quot/Quotient_Syntax.thy
changeset 1260 9df6144e281b
parent 1148 389d81959922
equal deleted inserted replaced
1259:db158e995bfc 1260:9df6144e281b
       
     1 (*  Title:      Quotient_Syntax.thy
       
     2     Author:     Cezary Kaliszyk and Christian Urban
       
     3 *)
       
     4 
       
     5 header {* Pretty syntax for Quotient operations *}
       
     6 
       
     7 (*<*)
       
     8 theory Quotient_Syntax
       
     9 imports Quotient
       
    10 begin
       
    11 
       
    12 notation
       
    13   rel_conj (infixr "OOO" 75) and
       
    14   fun_map (infixr "--->" 55) and
       
    15   fun_rel (infixr "===>" 55)
       
    16 
       
    17 end
       
    18 (*>*)