src/HOL/Word/TdThs.thy
changeset 27138 63fdfcf6c7a3
parent 27135 7fa9fa0bccee
child 29234 60f7fb56f8cd
--- a/src/HOL/Word/TdThs.thy	Tue Jun 10 21:50:30 2008 +0200
+++ b/src/HOL/Word/TdThs.thy	Tue Jun 10 23:28:35 2008 +0200
@@ -93,9 +93,11 @@
 interpretation nat_int: type_definition [int nat "Collect (op <= 0)"]
   by (rule td_nat_int)
 
-text "resetting to the default nat induct and cases rules"
-declare nat_induct [induct type: nat]
-declare nat.exhaust [cases type: nat]
+declare
+  nat_int.Rep_cases [cases del]
+  nat_int.Abs_cases [cases del]
+  nat_int.Rep_induct [induct del]
+  nat_int.Abs_induct [induct del]
 
 
 subsection "Extended form of type definition predicate"