src/HOL/Quotient_Examples/FSet.thy
changeset 57816 d8bbb97689d3
parent 55945 e96383acecf9
child 60515 484559628038
--- a/src/HOL/Quotient_Examples/FSet.thy	Thu Aug 07 12:17:41 2014 +0200
+++ b/src/HOL/Quotient_Examples/FSet.thy	Thu Aug 07 12:17:41 2014 +0200
@@ -985,7 +985,7 @@
   have b: "\<And>x' ys'. \<lbrakk>\<not> List.member ys' x'; a # xs \<approx> x' # ys'\<rbrakk> \<Longrightarrow> thesis" by fact
   have c: "xs = [] \<Longrightarrow> thesis" using b 
     apply(simp)
-    by (metis List.set_simps(1) emptyE empty_subsetI)
+    by (metis list.set(1) emptyE empty_subsetI)
   have "\<And>x ys. \<lbrakk>\<not> List.member ys x; xs \<approx> x # ys\<rbrakk> \<Longrightarrow> thesis"
   proof -
     fix x :: 'a