src/HOL/Library/BigO.thy
changeset 61585 a9599d3d7610
parent 60500 903bb1495239
child 61762 d50b993b4fb9
equal deleted inserted replaced
61584:f06e5a5a4b46 61585:a9599d3d7610
    14 O(h)$.  An earlier version of this library is described in detail in
    14 O(h)$.  An earlier version of this library is described in detail in
    15 @{cite "Avigad-Donnelly"}.
    15 @{cite "Avigad-Donnelly"}.
    16 
    16 
    17 The main changes in this version are as follows:
    17 The main changes in this version are as follows:
    18 \begin{itemize}
    18 \begin{itemize}
    19 \item We have eliminated the @{text O} operator on sets. (Most uses of this seem
    19 \item We have eliminated the \<open>O\<close> operator on sets. (Most uses of this seem
    20   to be inessential.)
    20   to be inessential.)
    21 \item We no longer use @{text "+"} as output syntax for @{text "+o"}
    21 \item We no longer use \<open>+\<close> as output syntax for \<open>+o\<close>
    22 \item Lemmas involving @{text "sumr"} have been replaced by more general lemmas
    22 \item Lemmas involving \<open>sumr\<close> have been replaced by more general lemmas
    23   involving `@{text "setsum"}.
    23   involving `\<open>setsum\<close>.
    24 \item The library has been expanded, with e.g.~support for expressions of
    24 \item The library has been expanded, with e.g.~support for expressions of
    25   the form @{text "f < g + O(h)"}.
    25   the form \<open>f < g + O(h)\<close>.
    26 \end{itemize}
    26 \end{itemize}
    27 
    27 
    28 Note also since the Big O library includes rules that demonstrate set
    28 Note also since the Big O library includes rules that demonstrate set
    29 inclusion, to use the automated reasoners effectively with the library
    29 inclusion, to use the automated reasoners effectively with the library
    30 one should redeclare the theorem @{text "subsetI"} as an intro rule,
    30 one should redeclare the theorem \<open>subsetI\<close> as an intro rule,
    31 rather than as an @{text "intro!"} rule, for example, using
    31 rather than as an \<open>intro!\<close> rule, for example, using
    32 \isa{\isakeyword{declare}}~@{text "subsetI [del, intro]"}.
    32 \isa{\isakeyword{declare}}~\<open>subsetI [del, intro]\<close>.
    33 \<close>
    33 \<close>
    34 
    34 
    35 subsection \<open>Definitions\<close>
    35 subsection \<open>Definitions\<close>
    36 
    36 
    37 definition bigo :: "('a \<Rightarrow> 'b::linordered_idom) \<Rightarrow> ('a \<Rightarrow> 'b) set"  ("(1O'(_'))")
    37 definition bigo :: "('a \<Rightarrow> 'b::linordered_idom) \<Rightarrow> ('a \<Rightarrow> 'b) set"  ("(1O'(_'))")