| changeset 67399 | eab6ce8368fa |
| parent 67339 | d91b9d22305b |
| child 67974 | 3f352a91b45a |
--- a/src/HOL/Analysis/Set_Integral.thy Wed Jan 10 15:21:49 2018 +0100 +++ b/src/HOL/Analysis/Set_Integral.thy Wed Jan 10 15:25:09 2018 +0100 @@ -310,7 +310,7 @@ by (auto intro!: set_integral_Un set_integrable_subset[OF f]) also have "\<dots> = (LINT x:A|M. f x) + (LINT x:B|M. f x)" using ae - by (intro arg_cong2[where f="op+"] set_integral_cong_set) + by (intro arg_cong2[where f="(+)"] set_integral_cong_set) (auto intro!: set_borel_measurable_subset[OF f']) finally show ?thesis . qed