src/HOL/Tools/Nitpick/nitpick_hol.ML
changeset 39557 fe5722fce758
parent 39360 cdf2c3341422
child 39687 4e9b6ada3a21
--- a/src/HOL/Tools/Nitpick/nitpick_hol.ML	Mon Sep 20 15:29:53 2010 +0200
+++ b/src/HOL/Tools/Nitpick/nitpick_hol.ML	Mon Sep 20 16:05:25 2010 +0200
@@ -1303,7 +1303,7 @@
       List.partition (is_typedef_axiom ctxt false) user_nondefs
       |>> append built_in_nondefs
     val defs =
-      (thy |> PureThy.all_thms_of
+      (thy |> Global_Theory.all_thms_of
            |> filter (curry (op =) Thm.definitionK o Thm.get_kind o snd)
            |> map (prop_of o snd)
            |> filter_out is_trivial_definition
@@ -1867,7 +1867,7 @@
 fun ground_theorem_table thy =
   fold ((fn @{const Trueprop} $ t1 =>
             is_ground_term t1 ? Inttab.map_default (hash_term t1, []) (cons t1)
-          | _ => I) o prop_of o snd) (PureThy.all_thms_of thy) Inttab.empty
+          | _ => I) o prop_of o snd) (Global_Theory.all_thms_of thy) Inttab.empty
 
 (* TODO: Move to "Nitpick.thy" *)
 val basic_ersatz_table =