Quot/Examples/IntEx.thy
changeset 632 d23416464f62
parent 625 5d6a2b5fb222
child 636 520a4084d064
--- a/Quot/Examples/IntEx.thy	Tue Dec 08 14:00:48 2009 +0100
+++ b/Quot/Examples/IntEx.thy	Tue Dec 08 16:35:40 2009 +0100
@@ -141,10 +141,10 @@
 done
 
 lemma "PLUS a b = PLUS a b"
-apply(tactic {* procedure_tac @{context} @{thm test1} 1 *})
-apply(tactic {* regularize_tac @{context} 1 *})
-apply(tactic {* all_inj_repabs_tac @{context} 1*})
-apply(tactic {* clean_tac @{context} 1 *}) 
+apply(lifting_setup rule: test1)
+apply(regularize)
+apply(injection)
+apply(cleaning)
 done
 
 thm lambda_prs