remove removed option
authorblanchet
Wed, 28 Apr 2010 16:47:56 +0200
changeset 36498 c36bbcb00689
parent 36497 d2e8e5561c35
child 36499 7ec5ceef117b
remove removed option
src/HOL/Metis_Examples/BigO.thy
--- a/src/HOL/Metis_Examples/BigO.thy	Wed Apr 28 16:15:45 2010 +0200
+++ b/src/HOL/Metis_Examples/BigO.thy	Wed Apr 28 16:47:56 2010 +0200
@@ -206,8 +206,6 @@
 qed
 
 
-sledgehammer_params [sorts]
-
 lemma bigo_alt_def: "O(f) = 
     {h. EX c. (0 < c & (ALL x. abs (h x) <= c * abs (f x)))}"
 by (auto simp add: bigo_def bigo_pos_const)