renamed lemma to a more consistent name
authorLars Hupel <lars.hupel@mytum.de>
Thu, 13 Oct 2016 15:43:15 +0200
changeset 64181 4d1d2de432fa
parent 64180 676763a9c269
child 64216 89514fa139c9
renamed lemma to a more consistent name
src/HOL/Library/Finite_Map.thy
--- a/src/HOL/Library/Finite_Map.thy	Thu Oct 13 14:41:45 2016 +0200
+++ b/src/HOL/Library/Finite_Map.thy	Thu Oct 13 15:43:15 2016 +0200
@@ -582,7 +582,7 @@
 lemma fmrel_on_fset_alt_def: "fmrel_on_fset S P m n \<longleftrightarrow> fBall S (\<lambda>x. rel_option P (fmlookup m x) (fmlookup n x))"
 by transfer' (auto simp: rel_map_on_set_def eq_onp_def rel_fun_def)
 
-lemma rel_map_on_fsetI[intro]:
+lemma fmrel_on_fsetI[intro]:
   assumes "\<And>x. x |\<in>| S \<Longrightarrow> rel_option P (fmlookup m x) (fmlookup n x)"
   shows "fmrel_on_fset S P m n"
 using assms