src/HOL/Num.thy
Mon, 02 Apr 2012 16:07:24 +0200 remove unnecessary qualifiers on names
Mon, 02 Apr 2012 16:06:24 +0200 add lemma Suc_1
Sun, 01 Apr 2012 16:09:58 +0200 removed Nat_Numeral.thy, moving all theorems elsewhere
Fri, 30 Mar 2012 16:44:23 +0200 load Tools/numeral.ML in Num.thy
Fri, 30 Mar 2012 16:43:07 +0200 tuned proof
Fri, 30 Mar 2012 15:56:12 +0200 set up numeral reorient simproc in Num.thy
Fri, 30 Mar 2012 12:32:35 +0200 replace lemmas eval_nat_numeral with a simpler reformulation
Fri, 30 Mar 2012 11:52:26 +0200 new lemmas for simplifying subtraction on nat numerals
Fri, 30 Mar 2012 10:41:27 +0200 move more theorems from Nat_Numeral.thy to Num.thy
Fri, 30 Mar 2012 08:15:29 +0200 fix search-and-replace errors
Fri, 30 Mar 2012 09:08:29 +0200 add constant pred_numeral k = numeral k - (1::nat);
Fri, 30 Mar 2012 08:10:28 +0200 move lemmas from Nat_Numeral to Int.thy and Num.thy
Thu, 29 Mar 2012 14:09:10 +0200 move many lemmas from Nat_Numeral.thy to Power.thy or Num.thy
Thu, 29 Mar 2012 11:47:30 +0200 bootstrap Num.thy before Power.thy;
Mon, 26 Mar 2012 20:07:29 +0200 fix incorrect code_modulename declarations
Sun, 25 Mar 2012 20:15:39 +0200 merged fork with new numeral representation (see NEWS)