src/HOL/Library/Quotient_Syntax.thy
author haftmann
Sun, 22 Jul 2012 09:56:34 +0200
changeset 49442 571cb1df0768
parent 40850 91e583511113
child 57287 e96383acecf9
permissions -rw-r--r--
library theories for debugging and parallel computing using code generation towards Isabelle/ML
     1 (*  Title:      HOL/Library/Quotient_Syntax.thy
     2     Author:     Cezary Kaliszyk and Christian Urban
     3 *)
     4 
     5 header {* Pretty syntax for Quotient operations *}
     6 
     7 theory Quotient_Syntax
     8 imports Main
     9 begin
    10 
    11 notation
    12   rel_conj (infixr "OOO" 75) and
    13   map_fun (infixr "--->" 55) and
    14   fun_rel (infixr "===>" 55)
    15 
    16 end