src/FOL/ex/LocaleTest.thy
changeset 26336 a0e2b706ce73
parent 26199 04817a8802f2
child 26343 0dd2eab7b296
equal deleted inserted replaced
26335:961bbcc9d85b 26336:a0e2b706ce73
    17 ML {* set show_sorts *}
    17 ML {* set show_sorts *}
    18 
    18 
    19 ML {*
    19 ML {*
    20   fun check_thm name = let
    20   fun check_thm name = let
    21     val thy = the_context ();
    21     val thy = the_context ();
    22     val thm = get_thm thy (Name name);
    22     val thm = get_thm thy (Facts.Named (name, NONE));
    23     val {prop, hyps, ...} = rep_thm thm;
    23     val {prop, hyps, ...} = rep_thm thm;
    24     val prems = Logic.strip_imp_prems prop;
    24     val prems = Logic.strip_imp_prems prop;
    25     val _ = if null hyps then ()
    25     val _ = if null hyps then ()
    26         else error ("Theorem " ^ quote name ^ " has meta hyps.\n" ^
    26         else error ("Theorem " ^ quote name ^ " has meta hyps.\n" ^
    27           "Consistency check of locales package failed.");
    27           "Consistency check of locales package failed.");