src/CCL/CCL.thy
changeset 60754 02924903a6fd
parent 59780 23b67731f4f0
child 60770 240563fbf41d
--- a/src/CCL/CCL.thy	Sat Jul 18 20:53:05 2015 +0200
+++ b/src/CCL/CCL.thy	Sat Jul 18 20:54:56 2015 +0200
@@ -268,7 +268,7 @@
   let
     fun mk_raw_dstnct_thm rls s =
       Goal.prove_global @{theory} [] [] (Syntax.read_prop_global @{theory} s)
-        (fn {context = ctxt, ...} => rtac @{thm notI} 1 THEN eresolve_tac ctxt rls 1)
+        (fn {context = ctxt, ...} => resolve_tac ctxt @{thms notI} 1 THEN eresolve_tac ctxt rls 1)
   in map (mk_raw_dstnct_thm caseB_lemmas)
     (mk_dstnct_rls @{theory} ["bot","true","false","pair","lambda"]) end