src/HOL/ex/Nominal2_Dummy.thy
changeset 58858 cc1e03929685
parent 58841 e16712bb1d41
parent 58857 b0ccc7e1e7f3
child 58859 d5ff8b782b29
equal deleted inserted replaced
58841:e16712bb1d41 58858:cc1e03929685
     1 header \<open>Dummy theory to anticipate AFP/Nominal2 keywords\<close>  (* Proof General legacy *)
       
     2 
       
     3 theory Nominal2_Dummy
       
     4 imports Main
       
     5 keywords
       
     6   "nominal_datatype" :: thy_decl and
       
     7   "nominal_function" "nominal_inductive" "nominal_termination" :: thy_goal and
       
     8   "atom_decl" "equivariance" :: thy_decl and
       
     9   "avoids" "binds"
       
    10 begin
       
    11 
       
    12 ML \<open>
       
    13 Outer_Syntax.command @{command_spec "nominal_datatype"} "dummy" Scan.fail;
       
    14 Outer_Syntax.command @{command_spec "nominal_function"} "dummy" Scan.fail;
       
    15 Outer_Syntax.command @{command_spec "nominal_inductive"} "dummy" Scan.fail;
       
    16 Outer_Syntax.command @{command_spec "nominal_termination"} "dummy" Scan.fail;
       
    17 Outer_Syntax.command @{command_spec "atom_decl"} "dummy" Scan.fail;
       
    18 Outer_Syntax.command @{command_spec "equivariance"} "dummy" Scan.fail;
       
    19 \<close>
       
    20 
       
    21 end
       
    22