src/HOL/Int.thy
changeset 59582 0fbed69ff081
parent 59556 aa2deef7cf47
child 59613 7103019278f0
equal deleted inserted replaced
59580:cbc38731d42f 59582:0fbed69ff081
   751 declaration {* K Int_Arith.setup *}
   751 declaration {* K Int_Arith.setup *}
   752 
   752 
   753 simproc_setup fast_arith ("(m::'a::linordered_idom) < n" |
   753 simproc_setup fast_arith ("(m::'a::linordered_idom) < n" |
   754   "(m::'a::linordered_idom) <= n" |
   754   "(m::'a::linordered_idom) <= n" |
   755   "(m::'a::linordered_idom) = n") =
   755   "(m::'a::linordered_idom) = n") =
   756   {* fn _ => fn ss => fn ct => Lin_Arith.simproc ss (term_of ct) *}
   756   {* fn _ => fn ss => fn ct => Lin_Arith.simproc ss (Thm.term_of ct) *}
   757 
   757 
   758 
   758 
   759 subsection{*More Inequality Reasoning*}
   759 subsection{*More Inequality Reasoning*}
   760 
   760 
   761 lemma zless_add1_eq: "(w < z + (1::int)) = (w<z | w=z)"
   761 lemma zless_add1_eq: "(w < z + (1::int)) = (w<z | w=z)"