src/HOL/Library/Set_Algebras.thy
changeset 61585 a9599d3d7610
parent 61337 4645502c3c64
child 63473 151bb79536a7
equal deleted inserted replaced
61584:f06e5a5a4b46 61585:a9599d3d7610
     9 begin
     9 begin
    10 
    10 
    11 text \<open>
    11 text \<open>
    12   This library lifts operations like addition and multiplication to
    12   This library lifts operations like addition and multiplication to
    13   sets.  It was designed to support asymptotic calculations. See the
    13   sets.  It was designed to support asymptotic calculations. See the
    14   comments at the top of theory @{text BigO}.
    14   comments at the top of theory \<open>BigO\<close>.
    15 \<close>
    15 \<close>
    16 
    16 
    17 instantiation set :: (plus) plus
    17 instantiation set :: (plus) plus
    18 begin
    18 begin
    19 
    19