src/HOL/ex/Adhoc_Overloading_Examples.thy
changeset 57507 a609065c9e15
parent 53538 4e9e150422d5
child 57512 cc97b347b301
--- a/src/HOL/ex/Adhoc_Overloading_Examples.thy	Fri Jul 04 15:46:13 2014 +0200
+++ b/src/HOL/ex/Adhoc_Overloading_Examples.thy	Fri Jul 04 15:50:28 2014 +0200
@@ -127,7 +127,8 @@
   apply (rule perms_imp_bij [OF f])
   apply (rule MOST_mono [OF perms_imp_MOST_eq [OF f]])
   apply (erule subst, rule inv_f_f)
-  by (rule bij_is_inj [OF perms_imp_bij [OF f]])
+  apply (rule bij_is_inj [OF perms_imp_bij [OF f]])
+  done
 
 lemma bij_Rep_perm: "bij (Rep_perm p)"
   using Rep_perm [of p] unfolding perms_def by simp
@@ -207,7 +208,11 @@
   PERMUTE permute_perm
 
 interpretation perm_permute: permute permute_perm
-  by (default) (simp add: diff_minus minus_add add_assoc permute_perm_def)+
+  apply default
+  unfolding permute_perm_def
+  apply simp
+  apply (simp only: diff_conv_add_uminus minus_add add_assoc)
+  done
 
 text {*Permuting functions.*}
 locale fun_permute =