src/HOL/Nominal/Examples/Pattern.thy
changeset 60580 7e741e22d7fc
parent 58889 5b7a9633cfa8
child 61069 aefe89038dd2
--- a/src/HOL/Nominal/Examples/Pattern.thy	Thu Jun 25 22:56:33 2015 +0200
+++ b/src/HOL/Nominal/Examples/Pattern.thy	Thu Jun 25 23:33:47 2015 +0200
@@ -62,20 +62,20 @@
   by (simp add: supp_def Collect_disj_eq del: disj_not1)
 
 instance pat :: pt_name
-proof intro_classes
-  case goal1
+proof (default, goals)
+  case (1 x)
   show ?case by (induct x) simp_all
 next
-  case goal2
+  case (2 _ _ x)
   show ?case by (induct x) (simp_all add: pt_name2)
 next
-  case goal3
+  case (3 _ _ x)
   then show ?case by (induct x) (simp_all add: pt_name3)
 qed
 
 instance pat :: fs_name
-proof intro_classes
-  case goal1
+proof (default, goals)
+  case (1 x)
   show ?case by (induct x) (simp_all add: fin_supp)
 qed