src/HOL/Library/Boolean_Algebra.thy
changeset 25594 43c718438f9f
parent 25283 c532fd8445a2
child 25691 8f8d83af100a
equal deleted inserted replaced
25593:0b0df6c8646a 25594:43c718438f9f
     6 *)
     6 *)
     7 
     7 
     8 header {* Boolean Algebras *}
     8 header {* Boolean Algebras *}
     9 
     9 
    10 theory Boolean_Algebra
    10 theory Boolean_Algebra
    11 imports Main
    11 imports PreList
    12 begin
    12 begin
    13 
    13 
    14 locale boolean =
    14 locale boolean =
    15   fixes conj :: "'a \<Rightarrow> 'a \<Rightarrow> 'a" (infixr "\<sqinter>" 70)
    15   fixes conj :: "'a \<Rightarrow> 'a \<Rightarrow> 'a" (infixr "\<sqinter>" 70)
    16   fixes disj :: "'a \<Rightarrow> 'a \<Rightarrow> 'a" (infixr "\<squnion>" 65)
    16   fixes disj :: "'a \<Rightarrow> 'a \<Rightarrow> 'a" (infixr "\<squnion>" 65)