src/HOL/TPTP/CASC_Setup.thy
changeset 44651 5d6a11e166cf
parent 44462 d9a657c44380
child 44890 22f665a2e91c
--- a/src/HOL/TPTP/CASC_Setup.thy	Fri Sep 02 14:43:20 2011 +0200
+++ b/src/HOL/TPTP/CASC_Setup.thy	Fri Sep 02 14:43:20 2011 +0200
@@ -131,7 +131,7 @@
                           Sledgehammer_Filter.no_relevance_override))
    ORELSE
    SOLVE_TIMEOUT (max_secs div 10) "metis"
-       (ALLGOALS (Metis_Tactics.metis_tac [] ctxt []))
+       (ALLGOALS (Metis_Tactic.metis_tac [] ctxt []))
    ORELSE
    SOLVE_TIMEOUT (max_secs div 10) "fast" (ALLGOALS (fast_tac ctxt))
    ORELSE