src/CTT/CTT.thy
changeset 58975 762ee71498fa
parent 58972 5b026cfc5f04
child 58976 b38a54bbfbd6
--- a/src/CTT/CTT.thy	Tue Nov 11 13:40:13 2014 +0100
+++ b/src/CTT/CTT.thy	Tue Nov 11 13:44:09 2014 +0100
@@ -480,7 +480,7 @@
 *}
 
 method_setup NE = {*
-  Scan.lift Args.name >> (fn s => fn ctxt => SIMPLE_METHOD' (NE_tac ctxt s))
+  Scan.lift Args.name_inner_syntax >> (fn s => fn ctxt => SIMPLE_METHOD' (NE_tac ctxt s))
 *}
 
 method_setup pc = {*