src/HOL/HOL.thy
changeset 9736 332fab43628f
parent 9713 2c5b42311eb0
child 9839 da5ca8b30244
--- a/src/HOL/HOL.thy	Tue Aug 29 22:31:36 2000 +0200
+++ b/src/HOL/HOL.thy	Wed Aug 30 10:21:19 2000 +0200
@@ -191,7 +191,7 @@
 
 (* theory and package setup *)
 
-use "HOL_lemmas.ML"	setup attrib_setup
+use "HOL_lemmas.ML"
 use "cladata.ML"	setup hypsubst_setup setup Classical.setup setup clasetup
 
 lemma all_eq: "(!!x. P x) == Trueprop (ALL x. P x)"
@@ -219,6 +219,6 @@
 use "simpdata.ML"	setup Simplifier.setup
 			setup "Simplifier.method_setup Splitter.split_modifiers" setup simpsetup
                         setup Splitter.setup setup Clasimp.setup setup iff_attrib_setup
-
+			setup attrib_setup
 
 end