src/CTT/ex/Typechecking.thy
changeset 39159 0dec18004e75
parent 36319 8feb2c4bef1a
child 58889 5b7a9633cfa8
--- a/src/CTT/ex/Typechecking.thy	Mon Sep 06 19:11:01 2010 +0200
+++ b/src/CTT/ex/Typechecking.thy	Mon Sep 06 19:13:10 2010 +0200
@@ -66,7 +66,7 @@
 
 (*Proofs involving arbitrary types.
   For concreteness, every type variable left over is forced to be N*)
-ML {* val N_tac = TRYALL (rtac (thm "NF")) *}
+ML {* val N_tac = TRYALL (rtac @{thm NF}) *}
 
 schematic_lemma "lam w. <w,w> : ?A"
 apply (tactic "typechk_tac []")