src/HOL/Topological_Spaces.thy
changeset 56518 beb3b6851665
parent 56371 fb9ae0727548
child 56524 f4ba736040fa
--- a/src/HOL/Topological_Spaces.thy	Thu Apr 10 17:48:13 2014 +0200
+++ b/src/HOL/Topological_Spaces.thy	Thu Apr 10 17:48:14 2014 +0200
@@ -2486,7 +2486,7 @@
 apply(auto simp add: rel_fun_def)
 done
 
-lemma left_total_rel_filter [reflexivity_rule]:
+lemma left_total_rel_filter [transfer_rule]:
   assumes [transfer_rule]: "bi_total A" "bi_unique A"
   shows "left_total (rel_filter A)"
 proof(rule left_totalI)
@@ -2511,7 +2511,7 @@
 unfolding bi_total_conv_left_right using assms
 by(simp add: left_total_rel_filter right_total_rel_filter)
 
-lemma left_unique_rel_filter [reflexivity_rule]:
+lemma left_unique_rel_filter [transfer_rule]:
   assumes "left_unique A"
   shows "left_unique (rel_filter A)"
 proof(rule left_uniqueI)