src/HOL/ex/Bubblesort.thy
changeset 66110 d59f9f696110
parent 63793 e68a0b651eb5
child 66453 cc19f7ca2ed6
--- a/src/HOL/ex/Bubblesort.thy	Sat Jun 17 15:41:19 2017 +0200
+++ b/src/HOL/ex/Bubblesort.thy	Sat Jun 17 18:49:19 2017 +0200
@@ -45,7 +45,7 @@
 apply(induction xs rule: bubble_min.induct)
   apply simp
  apply simp
-apply (auto simp: add_eq_conv_ex split: list.split)
+apply (auto split: list.split)
 done
 
 lemma bubble_minD_mset: