src/HOL/MicroJava/J/Example.thy
changeset 36319 8feb2c4bef1a
parent 35102 cc7a0b9f938c
child 45605 a89b4bc311a5
--- a/src/HOL/MicroJava/J/Example.thy	Fri Apr 23 23:33:48 2010 +0200
+++ b/src/HOL/MicroJava/J/Example.thy	Fri Apr 23 23:35:43 2010 +0200
@@ -371,7 +371,7 @@
 done
 
 ML {* val t = resolve_tac @{thms ty_expr_ty_exprs_wt_stmt.intros} 1 *}
-lemma wt_test: "(tprg, empty(e\<mapsto>Class Base))\<turnstile>  
+schematic_lemma wt_test: "(tprg, empty(e\<mapsto>Class Base))\<turnstile>  
   Expr(e::=NewC Ext);; Expr({Base}LAcc e..foo({?pTs'}[Lit Null]))\<surd>"
 apply (tactic t) -- ";;"
 apply  (tactic t) -- "Expr"
@@ -400,7 +400,7 @@
 
 declare split_if [split del]
 declare init_vars_def [simp] c_hupd_def [simp] cast_ok_def [simp]
-lemma exec_test: 
+schematic_lemma exec_test: 
 " [|new_Addr (heap (snd s0)) = (a, None)|] ==>  
   tprg\<turnstile>s0 -test-> ?s"
 apply (unfold test_def)