Theory Nominal2_Dummy

theory Nominal2_Dummy
imports Main
header ‹Dummy theory to anticipate AFP/Nominal2 keywords›  (* 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 ‹
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;
›

end