src/HOL/Nominal/Examples/Class.thy
changeset 22542 8279a25ad0ae
parent 22418 49e2d9744ae1
child 23092 f3615235dc4d
--- a/src/HOL/Nominal/Examples/Class.thy	Wed Mar 28 18:25:23 2007 +0200
+++ b/src/HOL/Nominal/Examples/Class.thy	Wed Mar 28 19:16:11 2007 +0200
@@ -35,7 +35,7 @@
 
 text {* Induction principles *}
 
-thm trm.induct_weak --"weak"
+thm trm.weak_induct --"weak"
 thm trm.induct      --"strong"
 thm trm.induct'     --"strong with explicit context (rarely needed)"