src/HOL/Fields.thy
changeset 57950 59c17b0b870d
parent 57514 bdc2c6b40bf2
child 58512 dc4d76dfa8f0
--- a/src/HOL/Fields.thy	Sat Aug 16 13:54:19 2014 +0200
+++ b/src/HOL/Fields.thy	Sat Aug 16 14:12:39 2014 +0200
@@ -25,15 +25,7 @@
 
 text{* Lemmas @{text divide_simps} move division to the outside and eliminates them on (in)equalities. *}
 
-ML {*
-structure Divide_Simps = Named_Thms
-(
-  val name = @{binding divide_simps}
-  val description = "rewrite rules to eliminate divisions"
-)
-*}
-
-setup Divide_Simps.setup
+named_theorems divide_simps "rewrite rules to eliminate divisions"
 
 
 class division_ring = ring_1 + inverse +