src/HOL/Lattices_Big.thy
changeset 55089 181751ad852f
parent 54868 bab6cade3cc5
child 55803 74d3fe9031d8
equal deleted inserted replaced
55088:57c82e01022b 55089:181751ad852f
     4 *)
     4 *)
     5 
     5 
     6 header {* Big infimum (minimum) and supremum (maximum) over finite (non-empty) sets *}
     6 header {* Big infimum (minimum) and supremum (maximum) over finite (non-empty) sets *}
     7 
     7 
     8 theory Lattices_Big
     8 theory Lattices_Big
     9 imports Finite_Set
     9 imports Finite_Set Option
    10 begin
    10 begin
    11 
    11 
    12 subsection {* Generic lattice operations over a set *}
    12 subsection {* Generic lattice operations over a set *}
    13 
    13 
    14 no_notation times (infixl "*" 70)
    14 no_notation times (infixl "*" 70)