src/HOL/ex/Nominal2_Dummy.thy
changeset 57064 8a1be5efe628
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/ex/Nominal2_Dummy.thy	Thu May 22 15:49:36 2014 +0200
@@ -0,0 +1,22 @@
+header \<open>Dummy theory to anticipate AFP/Nominal2 keywords\<close>  (* Proof General legacy *)
+
+theory Nominal2_Dummy
+imports Main
+keywords
+  "nominal_datatype" :: thy_decl and
+  "nominal_function" "nominal_inductive" "nominal_termination" :: thy_goal and
+  "atom_decl" "equivariance" :: thy_decl and
+  "avoids" "binds"
+begin
+
+ML \<open>
+Outer_Syntax.command @{command_spec "nominal_datatype"} "dummy" Scan.fail;
+Outer_Syntax.command @{command_spec "nominal_function"} "dummy" Scan.fail;
+Outer_Syntax.command @{command_spec "nominal_inductive"} "dummy" Scan.fail;
+Outer_Syntax.command @{command_spec "nominal_termination"} "dummy" Scan.fail;
+Outer_Syntax.command @{command_spec "atom_decl"} "dummy" Scan.fail;
+Outer_Syntax.command @{command_spec "equivariance"} "dummy" Scan.fail;
+\<close>
+
+end
+