src/FOL/ex/Locale_Test/Locale_Test1.thy
changeset 80866 8c67b14fdd48
parent 78031 a526f69145ec
equal deleted inserted replaced
80865:7c20c207af48 80866:8c67b14fdd48
   130 
   130 
   131 ML \<open>
   131 ML \<open>
   132   fun check_syntax ctxt thm expected =
   132   fun check_syntax ctxt thm expected =
   133     let
   133     let
   134       val obtained =
   134       val obtained =
   135         Print_Mode.setmp [] (Thm.string_of_thm (Config.put show_markup false ctxt)) thm;
   135         Pretty.pure_string_of (Thm.pretty_thm (Config.put show_markup false ctxt) thm);
   136     in
   136     in
   137       if obtained <> expected
   137       if obtained <> expected
   138       then error ("Theorem syntax '" ^ obtained ^ "' obtained, but '" ^ expected ^ "' expected.")
   138       then error ("Theorem syntax '" ^ obtained ^ "' obtained, but '" ^ expected ^ "' expected.")
   139       else ()
   139       else ()
   140     end;
   140     end;