src/HOL/Nitpick_Examples/Mono_Nits.thy
changeset 77889 5db014c36f42
parent 74399 a1d33d1bfb6d
child 77892 44d845b15214
--- a/src/HOL/Nitpick_Examples/Mono_Nits.thy	Wed Apr 19 23:27:55 2023 +0200
+++ b/src/HOL/Nitpick_Examples/Mono_Nits.thy	Thu Apr 20 11:57:34 2023 +0200
@@ -153,7 +153,7 @@
 fun theorems_of thy =
   filter (fn (name, th) =>
              not (is_forbidden_theorem name) andalso
-             Thm.theory_name th = Context.theory_name thy)
+             Thm.theory_base_name th = Context.theory_base_name thy)
          (Global_Theory.all_thms_of thy true)
 
 fun check_formulas tsp =
@@ -175,7 +175,7 @@
 
 fun check_theory thy =
   let
-    val path = File.tmp_path (Context.theory_name thy ^ ".out" |> Path.explode)
+    val path = File.tmp_path (Context.theory_base_name thy ^ ".out" |> Path.explode)
     val _ = File.write path ""
     fun check_theorem (name, th) =
       let