src/HOL/Library/Numeral_Type.thy
changeset 29999 da85a244e328
parent 29998 19e1ef628b25
child 30001 dd27e16677b2
--- a/src/HOL/Library/Numeral_Type.thy	Thu Feb 19 17:11:12 2009 -0800
+++ b/src/HOL/Library/Numeral_Type.thy	Thu Feb 19 17:13:35 2009 -0800
@@ -347,11 +347,11 @@
 
 text {* Set up cases, induction, and arithmetic *}
 
-lemmas bit0_cases [cases type: bit0, case_names of_int] = bit0.cases
-lemmas bit1_cases [cases type: bit1, case_names of_int] = bit1.cases
+lemmas bit0_cases [case_names of_int, cases type: bit0] = bit0.cases
+lemmas bit1_cases [case_names of_int, cases type: bit1] = bit1.cases
 
-lemmas bit0_induct [induct type: bit0, case_names of_int] = bit0.induct
-lemmas bit1_induct [induct type: bit1, case_names of_int] = bit1.induct
+lemmas bit0_induct [case_names of_int, induct type: bit0] = bit0.induct
+lemmas bit1_induct [case_names of_int, induct type: bit1] = bit1.induct
 
 lemmas bit0_iszero_number_of [simp] = bit0.iszero_number_of
 lemmas bit1_iszero_number_of [simp] = bit1.iszero_number_of