src/HOL/ex/Set_Comprehension_Pointfree_Examples.thy
changeset 61337 4645502c3c64
parent 58889 5b7a9633cfa8
child 61343 5b5656a63bd6
--- a/src/HOL/ex/Set_Comprehension_Pointfree_Examples.thy	Tue Oct 06 13:31:44 2015 +0200
+++ b/src/HOL/ex/Set_Comprehension_Pointfree_Examples.thy	Tue Oct 06 15:14:28 2015 +0200
@@ -111,7 +111,7 @@
 using assms by (auto intro!: finite_vimageI simp add: inj_on_def)
   (* injectivity to be automated with further rules and automation *)
 
-schematic_lemma (* check interaction with schematics *)
+schematic_goal (* check interaction with schematics *)
   "finite {x :: ?'A \<Rightarrow> ?'B \<Rightarrow> bool. \<exists>a b. x = Pair_Rep a b}
    = finite ((\<lambda>(b :: ?'B, a:: ?'A). Pair_Rep a b) ` (UNIV \<times> UNIV))"
   by simp