src/HOL/Nitpick_Examples/Refute_Nits.thy
changeset 61337 4645502c3c64
parent 61076 bdc1e2f0a86a
child 62145 5b946c81dfbf
--- a/src/HOL/Nitpick_Examples/Refute_Nits.thy	Tue Oct 06 13:31:44 2015 +0200
+++ b/src/HOL/Nitpick_Examples/Refute_Nits.thy	Tue Oct 06 15:14:28 2015 +0200
@@ -340,12 +340,12 @@
 
 subsubsection {* Schematic Variables *}
 
-schematic_lemma "?P"
+schematic_goal "?P"
 nitpick [expect = none]
 apply auto
 done
 
-schematic_lemma "x = ?y"
+schematic_goal "x = ?y"
 nitpick [expect = none]
 apply auto
 done