src/FOL/ex/Classical.thy
changeset 36319 8feb2c4bef1a
parent 32960 69916a850301
child 42789 3a84b6947932
--- a/src/FOL/ex/Classical.thy	Fri Apr 23 23:33:48 2010 +0200
+++ b/src/FOL/ex/Classical.thy	Fri Apr 23 23:35:43 2010 +0200
@@ -363,7 +363,7 @@
 
 text{*Non-equational version, from Manthey and Bry, CADE-9 (Springer, 1988).
   fast DISCOVERS who killed Agatha. *}
-lemma "lives(agatha) & lives(butler) & lives(charles) &  
+schematic_lemma "lives(agatha) & lives(butler) & lives(charles) &  
    (killed(agatha,agatha) | killed(butler,agatha) | killed(charles,agatha)) &  
    (\<forall>x y. killed(x,y) --> hates(x,y) & ~richer(x,y)) &  
    (\<forall>x. hates(agatha,x) --> ~hates(charles,x)) &