src/HOL/ex/Fundefs.thy
changeset 39754 150f831ce4a3
parent 36270 fd95c0514623
child 40111 80b7f456600f
--- a/src/HOL/ex/Fundefs.thy	Tue Sep 28 09:43:13 2010 +0200
+++ b/src/HOL/ex/Fundefs.thy	Tue Sep 28 09:54:07 2010 +0200
@@ -51,7 +51,7 @@
   assumes trm: "nz_dom x"
   shows "nz x = 0"
 using trm
-by induct auto
+by induct (auto simp: nz.psimps)
 
 termination nz
   by (relation "less_than") (auto simp:nz_is_zero)
@@ -71,7 +71,7 @@
 lemma f91_estimate: 
   assumes trm: "f91_dom n"
   shows "n < f91 n + 11"
-using trm by induct auto
+using trm by induct (auto simp: f91.psimps)
 
 termination
 proof