src/HOL/Int.thy
changeset 30796 126701134811
parent 30652 752329615264
child 30802 f9e9e800d27e
equal deleted inserted replaced
30794:787b39d499cf 30796:126701134811
    10 theory Int
    10 theory Int
    11 imports Equiv_Relations Nat Wellfounded
    11 imports Equiv_Relations Nat Wellfounded
    12 uses
    12 uses
    13   ("Tools/numeral.ML")
    13   ("Tools/numeral.ML")
    14   ("Tools/numeral_syntax.ML")
    14   ("Tools/numeral_syntax.ML")
    15   ("~~/src/Provers/Arith/assoc_fold.ML")
    15   "~~/src/Provers/Arith/assoc_fold.ML"
    16   "~~/src/Provers/Arith/cancel_numerals.ML"
    16   "~~/src/Provers/Arith/cancel_numerals.ML"
    17   "~~/src/Provers/Arith/combine_numerals.ML"
    17   "~~/src/Provers/Arith/combine_numerals.ML"
    18   ("Tools/int_arith.ML")
    18   ("Tools/int_arith.ML")
    19 begin
    19 begin
    20 
    20 
  1523 text {* Legacy theorems *}
  1523 text {* Legacy theorems *}
  1524 
  1524 
  1525 lemmas zle_int = of_nat_le_iff [where 'a=int]
  1525 lemmas zle_int = of_nat_le_iff [where 'a=int]
  1526 lemmas int_int_eq = of_nat_eq_iff [where 'a=int]
  1526 lemmas int_int_eq = of_nat_eq_iff [where 'a=int]
  1527 
  1527 
  1528 use "~~/src/Provers/Arith/assoc_fold.ML"
       
  1529 use "Tools/int_arith.ML"
  1528 use "Tools/int_arith.ML"
  1530 declaration {* K Int_Arith.setup *}
  1529 declaration {* K Int_Arith.setup *}
  1531 
  1530 
  1532 
  1531 
  1533 subsection{*Lemmas About Small Numerals*}
  1532 subsection{*Lemmas About Small Numerals*}