src/HOL/Library/Quotient_Syntax.thy
changeset 35222 4f1fba00f66d
child 35787 afdf1c4958b2
equal deleted inserted replaced
35221:5cb63cb4213f 35222:4f1fba00f66d
       
     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 Main
       
    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 (*>*)