src/HOL/Tools/Nitpick/nitpick_hol.ML
changeset 39557 fe5722fce758
parent 39360 cdf2c3341422
child 39687 4e9b6ada3a21
equal deleted inserted replaced
39556:32a00ff29d1a 39557:fe5722fce758
  1301       partition_axioms_by_definitionality ctxt user_axioms def_names
  1301       partition_axioms_by_definitionality ctxt user_axioms def_names
  1302     val (built_in_nondefs, user_nondefs) =
  1302     val (built_in_nondefs, user_nondefs) =
  1303       List.partition (is_typedef_axiom ctxt false) user_nondefs
  1303       List.partition (is_typedef_axiom ctxt false) user_nondefs
  1304       |>> append built_in_nondefs
  1304       |>> append built_in_nondefs
  1305     val defs =
  1305     val defs =
  1306       (thy |> PureThy.all_thms_of
  1306       (thy |> Global_Theory.all_thms_of
  1307            |> filter (curry (op =) Thm.definitionK o Thm.get_kind o snd)
  1307            |> filter (curry (op =) Thm.definitionK o Thm.get_kind o snd)
  1308            |> map (prop_of o snd)
  1308            |> map (prop_of o snd)
  1309            |> filter_out is_trivial_definition
  1309            |> filter_out is_trivial_definition
  1310            |> filter is_plain_definition) @
  1310            |> filter is_plain_definition) @
  1311       user_defs @ built_in_defs
  1311       user_defs @ built_in_defs
  1865   end
  1865   end
  1866 
  1866 
  1867 fun ground_theorem_table thy =
  1867 fun ground_theorem_table thy =
  1868   fold ((fn @{const Trueprop} $ t1 =>
  1868   fold ((fn @{const Trueprop} $ t1 =>
  1869             is_ground_term t1 ? Inttab.map_default (hash_term t1, []) (cons t1)
  1869             is_ground_term t1 ? Inttab.map_default (hash_term t1, []) (cons t1)
  1870           | _ => I) o prop_of o snd) (PureThy.all_thms_of thy) Inttab.empty
  1870           | _ => I) o prop_of o snd) (Global_Theory.all_thms_of thy) Inttab.empty
  1871 
  1871 
  1872 (* TODO: Move to "Nitpick.thy" *)
  1872 (* TODO: Move to "Nitpick.thy" *)
  1873 val basic_ersatz_table =
  1873 val basic_ersatz_table =
  1874   [(@{const_name card}, @{const_name card'}),
  1874   [(@{const_name card}, @{const_name card'}),
  1875    (@{const_name setsum}, @{const_name setsum'}),
  1875    (@{const_name setsum}, @{const_name setsum'}),