changeset 22187 | a2c4861363d5 |
parent 21834 | 770ce948a59b |
child 22473 | 753123c89d72 |
--- a/src/HOL/Integ/Numeral.thy Thu Jan 25 09:32:56 2007 +0100 +++ b/src/HOL/Integ/Numeral.thy Thu Jan 25 16:57:57 2007 +0100 @@ -74,6 +74,11 @@ pred :: "int \<Rightarrow> int" where "pred k = k - 1" +declare + max_def[of "number_of u" "number_of v", standard, simp] + min_def[of "number_of u" "number_of v", standard, simp] + -- {* unfolding @{text minx} and @{text max} on numerals *} + lemmas numeral_simps = succ_def pred_def Pls_def Min_def Bit_def