src/HOL/Library/BigO.thy
changeset 63485 ea8dfb0ed10e
parent 63473 151bb79536a7
child 63918 6bf55e6e0b75
--- a/src/HOL/Library/BigO.thy	Wed Jul 13 20:14:16 2016 +0200
+++ b/src/HOL/Library/BigO.thy	Wed Jul 13 20:47:56 2016 +0200
@@ -5,7 +5,10 @@
 section \<open>Big O notation\<close>
 
 theory BigO
-  imports Complex_Main Function_Algebras Set_Algebras
+  imports
+    Complex_Main
+    Function_Algebras
+    Set_Algebras
 begin
 
 text \<open>