src/HOL/Prolog/Func.thy
changeset 61337 4645502c3c64
parent 58889 5b7a9633cfa8
child 63167 0909deb8059b
--- a/src/HOL/Prolog/Func.thy	Tue Oct 06 13:31:44 2015 +0200
+++ b/src/HOL/Prolog/Func.thy	Tue Oct 06 15:14:28 2015 +0200
@@ -58,11 +58,11 @@
 
 lemmas prog_Func = eval
 
-schematic_lemma "eval ((S (S Z)) + (S Z)) ?X"
+schematic_goal "eval ((S (S Z)) + (S Z)) ?X"
   apply (prolog prog_Func)
   done
 
-schematic_lemma "eval (app (fix (%fact. abs(%n. cond (n eq Z) (S Z)
+schematic_goal "eval (app (fix (%fact. abs(%n. cond (n eq Z) (S Z)
                         (n * (app fact (n - (S Z))))))) (S (S (S Z)))) ?X"
   apply (prolog prog_Func)
   done