diff -r a80d8ec6c998 -r 3dda49e08b9d src/HOL/Semiring_Normalization.thy --- a/src/HOL/Semiring_Normalization.thy Fri Jan 04 21:49:06 2019 +0100 +++ b/src/HOL/Semiring_Normalization.thy Fri Jan 04 23:22:53 2019 +0100 @@ -114,7 +114,7 @@ local_setup \ Semiring_Normalizer.declare @{thm comm_semiring_1_axioms} - {semiring = ([@{term "x + y"}, @{term "x * y"}, @{term "x ^ n"}, @{term 0}, @{term 1}], + {semiring = ([\<^term>\x + y\, \<^term>\x * y\, \<^term>\x ^ n\, \<^term>\0\, \<^term>\1\], @{thms semiring_normalization_rules}), ring = ([], []), field = ([], []), @@ -134,9 +134,9 @@ local_setup \ Semiring_Normalizer.declare @{thm comm_ring_1_axioms} - {semiring = ([@{term "x + y"}, @{term "x * y"}, @{term "x ^ n"}, @{term 0}, @{term 1}], + {semiring = ([\<^term>\x + y\, \<^term>\x * y\, \<^term>\x ^ n\, \<^term>\0\, \<^term>\1\], @{thms semiring_normalization_rules}), - ring = ([@{term "x - y"}, @{term "- x"}], @{thms ring_normalization_rules}), + ring = ([\<^term>\x - y\, \<^term>\- x\], @{thms ring_normalization_rules}), field = ([], []), idom = [], ideal = []} @@ -149,7 +149,7 @@ local_setup \ Semiring_Normalizer.declare @{thm comm_semiring_1_cancel_crossproduct_axioms} - {semiring = ([@{term "x + y"}, @{term "x * y"}, @{term "x ^ n"}, @{term 0}, @{term 1}], + {semiring = ([\<^term>\x + y\, \<^term>\x * y\, \<^term>\x ^ n\, \<^term>\0\, \<^term>\1\], @{thms semiring_normalization_rules}), ring = ([], []), field = ([], []), @@ -164,9 +164,9 @@ local_setup \ Semiring_Normalizer.declare @{thm idom_axioms} - {semiring = ([@{term "x + y"}, @{term "x * y"}, @{term "x ^ n"}, @{term 0}, @{term 1}], + {semiring = ([\<^term>\x + y\, \<^term>\x * y\, \<^term>\x ^ n\, \<^term>\0\, \<^term>\1\], @{thms semiring_normalization_rules}), - ring = ([@{term "x - y"}, @{term "- x"}], @{thms ring_normalization_rules}), + ring = ([\<^term>\x - y\, \<^term>\- x\], @{thms ring_normalization_rules}), field = ([], []), idom = @{thms crossproduct_noteq add_scale_eq_noteq}, ideal = @{thms right_minus_eq add_0_iff}} @@ -179,10 +179,10 @@ local_setup \ Semiring_Normalizer.declare @{thm field_axioms} - {semiring = ([@{term "x + y"}, @{term "x * y"}, @{term "x ^ n"}, @{term 0}, @{term 1}], + {semiring = ([\<^term>\x + y\, \<^term>\x * y\, \<^term>\x ^ n\, \<^term>\0\, \<^term>\1\], @{thms semiring_normalization_rules}), - ring = ([@{term "x - y"}, @{term "- x"}], @{thms ring_normalization_rules}), - field = ([@{term "x / y"}, @{term "inverse x"}], @{thms divide_inverse inverse_eq_divide}), + ring = ([\<^term>\x - y\, \<^term>\- x\], @{thms ring_normalization_rules}), + field = ([\<^term>\x / y\, \<^term>\inverse x\], @{thms divide_inverse inverse_eq_divide}), idom = @{thms crossproduct_noteq add_scale_eq_noteq}, ideal = @{thms right_minus_eq add_0_iff}} \