src/HOL/Library/RBT_Set.thy
changeset 67682 00c436488398
parent 67408 4a4c14b24800
child 68109 cebf36c14226
--- a/src/HOL/Library/RBT_Set.thy	Tue Feb 20 22:04:04 2018 +0100
+++ b/src/HOL/Library/RBT_Set.thy	Tue Feb 20 22:25:23 2018 +0100
@@ -474,7 +474,7 @@
 proof -
   interpret comp_fun_idem Set.insert
     by (fact comp_fun_idem_insert)
-  from finite_fold_fold_keys[OF \<open>comp_fun_commute Set.insert\<close>]
+  from finite_fold_fold_keys[OF comp_fun_commute_axioms]
   show ?thesis by (auto simp add: union_fold_insert)
 qed
 
@@ -487,7 +487,7 @@
 proof -
   interpret comp_fun_idem Set.remove
     by (fact comp_fun_idem_remove)
-  from finite_fold_fold_keys[OF \<open>comp_fun_commute Set.remove\<close>]
+  from finite_fold_fold_keys[OF comp_fun_commute_axioms]
   show ?thesis by (auto simp add: minus_fold_remove)
 qed