src/HOL/Analysis/Henstock_Kurzweil_Integration.thy
changeset 68403 223172b97d0b
parent 68361 20375f232f3b
child 68527 2f4e2aab190a
--- a/src/HOL/Analysis/Henstock_Kurzweil_Integration.thy	Wed Jun 06 13:04:52 2018 +0200
+++ b/src/HOL/Analysis/Henstock_Kurzweil_Integration.thy	Wed Jun 06 18:19:55 2018 +0200
@@ -772,13 +772,13 @@
   fixes f :: "_ \<Rightarrow> 'b :: real_normed_field"
   assumes "f integrable_on s"
   shows "(\<lambda>x. f x / of_real c) integrable_on s"
-by (simp add: integrable_on_cmult_right divide_inverse assms reorient: of_real_inverse)
+by (simp add: integrable_on_cmult_right divide_inverse assms flip: of_real_inverse)
 
 lemma integrable_on_cdivide_iff [simp]:
   fixes f :: "_ \<Rightarrow> 'b :: real_normed_field"
   assumes "c \<noteq> 0"
   shows "(\<lambda>x. f x / of_real c) integrable_on s \<longleftrightarrow> f integrable_on s"
-by (simp add: divide_inverse assms reorient: of_real_inverse)
+by (simp add: divide_inverse assms flip: of_real_inverse)
 
 lemma has_integral_null [intro]: "content(cbox a b) = 0 \<Longrightarrow> (f has_integral 0) (cbox a b)"
   unfolding has_integral_cbox
@@ -3410,7 +3410,7 @@
       by (simp add: inner_simps field_simps)
     ultimately show ?thesis using False
       by (simp add: image_affinity_cbox content_cbox'
-        prod.distrib[symmetric] inner_diff_left reorient: prod_constant)
+        prod.distrib[symmetric] inner_diff_left flip: prod_constant)
   qed
 qed