src/HOL/Library/Predicate_Compile_Alternative_Defs.thy
changeset 54489 03ff4d1e6784
parent 51143 0a2371e7ced3
child 55414 eab03e9cee8a
equal deleted inserted replaced
54488:b60f1fab408c 54489:03ff4d1e6784
    43   "A = B \<longleftrightarrow> (\<forall>x. A x \<longrightarrow> B x) \<and> (\<forall>x. B x \<longrightarrow> A x)"
    43   "A = B \<longleftrightarrow> (\<forall>x. A x \<longrightarrow> B x) \<and> (\<forall>x. B x \<longrightarrow> A x)"
    44   by (auto simp add: fun_eq_iff)
    44   by (auto simp add: fun_eq_iff)
    45 
    45 
    46 section {* Setup for Numerals *}
    46 section {* Setup for Numerals *}
    47 
    47 
    48 setup {* Predicate_Compile_Data.ignore_consts [@{const_name numeral}, @{const_name neg_numeral}] *}
    48 setup {* Predicate_Compile_Data.ignore_consts [@{const_name numeral}] *}
    49 setup {* Predicate_Compile_Data.keep_functions [@{const_name numeral}, @{const_name neg_numeral}] *}
    49 setup {* Predicate_Compile_Data.keep_functions [@{const_name numeral}] *}
    50 
    50 
    51 setup {* Predicate_Compile_Data.ignore_consts [@{const_name div}, @{const_name mod}, @{const_name times}] *}
    51 setup {* Predicate_Compile_Data.ignore_consts [@{const_name div}, @{const_name mod}, @{const_name times}] *}
    52 
    52 
    53 section {* Arithmetic operations *}
    53 section {* Arithmetic operations *}
    54 
    54