| changeset 48891 | c0eafbd55de3 | 
| parent 47701 | 157e6108a342 | 
| child 55926 | 3ef14caf5637 | 
--- a/src/HOL/Algebra/Ring.thy Wed Aug 22 22:47:16 2012 +0200 +++ b/src/HOL/Algebra/Ring.thy Wed Aug 22 22:55:41 2012 +0200 @@ -5,7 +5,6 @@ theory Ring imports FiniteProduct -uses ("ringsimp.ML") begin section {* The Algebraic Hierarchy of Rings *} @@ -389,7 +388,7 @@ text {* Setup algebra method: compute distributive normal form in locale contexts *} -use "ringsimp.ML" +ML_file "ringsimp.ML" setup Algebra.attrib_setup