src/HOL/Semiring_Normalization.thy
changeset 58826 2ed2eaabe3df
parent 57514 bdc2c6b40bf2
child 58889 5b7a9633cfa8
--- a/src/HOL/Semiring_Normalization.thy	Wed Oct 29 17:01:44 2014 +0100
+++ b/src/HOL/Semiring_Normalization.thy	Wed Oct 29 19:01:49 2014 +0100
@@ -8,8 +8,6 @@
 imports Numeral_Simprocs Nat_Transfer
 begin
 
-ML_file "Tools/semiring_normalizer.ML"
-
 text {* Prelude *}
 
 class comm_semiring_1_cancel_crossproduct = comm_semiring_1_cancel +
@@ -69,7 +67,7 @@
 
 text {* Semiring normalization proper *}
 
-setup Semiring_Normalizer.setup
+ML_file "Tools/semiring_normalizer.ML"
 
 context comm_semiring_1
 begin