src/HOL/Quotient_Examples/Quotient_Int.thy
changeset 40928 ace26e2cee91
parent 40468 d4aac200199e
child 41413 64cd30d6b0b8
--- a/src/HOL/Quotient_Examples/Quotient_Int.thy	Fri Dec 03 09:58:32 2010 +0100
+++ b/src/HOL/Quotient_Examples/Quotient_Int.thy	Fri Dec 03 10:03:10 2010 +0100
@@ -275,7 +275,7 @@
 proof (cases x, clarify)
   fix a b
   show "P (a, b)"
-  proof (induct a arbitrary: b rule: Nat.induct)
+  proof (induct a arbitrary: b rule: nat.induct)
     case zero
     show "P (0, b)" using assms by (induct b) auto
   next