src/HOL/Finite_Set.thy
changeset 17085 5b57f995a179
parent 17022 b257300c3a9c
child 17149 e2b19c92ef51
--- a/src/HOL/Finite_Set.thy	Tue Aug 16 15:36:28 2005 +0200
+++ b/src/HOL/Finite_Set.thy	Tue Aug 16 18:53:11 2005 +0200
@@ -2256,14 +2256,17 @@
 text{* Now we instantiate the recursion equations and declare them
 simplification rules: *}
 
-(* Making Min (resp. Max) a defined parameter of a locale suitably
-  extending ACIf could make the following interpretations more automatic. *)
+(* Making Min or Max a defined parameter of a locale, suitably
+  extending ACIf, could make the following interpretations more automatic. *)
 
-declare
-  fold1_singleton_def[OF Min_def, simp]
-  min.fold1_insert_idem_def[OF Min_def, simp]
-  fold1_singleton_def[OF Max_def, simp]
-  max.fold1_insert_idem_def[OF Max_def, simp]
+lemmas Min_singleton = fold1_singleton_def [OF Min_def]
+lemmas Max_singleton = fold1_singleton_def [OF Max_def]
+lemmas Min_insert = min.fold1_insert_idem_def [OF Min_def]
+lemmas Max_insert = max.fold1_insert_idem_def [OF Max_def]
+
+declare Min_singleton [simp]  Max_singleton [simp]
+declare Min_insert [simp]  Max_insert [simp]
+
 
 text{* Now we instantiate some @{text fold1} properties: *}