src/HOL/Nominal/Nominal.thy
changeset 19986 3e0eababf58d
parent 19972 89c5afe4139a
child 20388 b5a61270ea5a
equal deleted inserted replaced
19985:d39c554cf750 19986:3e0eababf58d
  2933 
  2933 
  2934 (***************************************)
  2934 (***************************************)
  2935 (* setup for the individial atom-kinds *)
  2935 (* setup for the individial atom-kinds *)
  2936 (* and nominal datatypes               *)
  2936 (* and nominal datatypes               *)
  2937 use "nominal_atoms.ML"
  2937 use "nominal_atoms.ML"
       
  2938 (* permutation equality tactic *)
       
  2939 use "nominal_permeq.ML";
  2938 use "nominal_package.ML"
  2940 use "nominal_package.ML"
  2939 setup "NominalAtoms.setup"
  2941 setup "NominalAtoms.setup"
  2940 
  2942 
  2941 (*****************************************)
  2943 (*****************************************)
  2942 (* setup for induction principles method *)
  2944 (* setup for induction principles method *)
  2944 use "nominal_induct.ML";
  2946 use "nominal_induct.ML";
  2945 method_setup nominal_induct =
  2947 method_setup nominal_induct =
  2946   {* NominalInduct.nominal_induct_method *}
  2948   {* NominalInduct.nominal_induct_method *}
  2947   {* nominal induction *}
  2949   {* nominal induction *}
  2948 
  2950 
  2949 (*******************************)
       
  2950 (* permutation equality tactic *)
       
  2951 use "nominal_permeq.ML";
       
  2952 
       
  2953 method_setup perm_simp =
  2951 method_setup perm_simp =
  2954   {* perm_eq_meth *}
  2952   {* NominalPermeq.perm_eq_meth *}
  2955   {* simp rules and simprocs for analysing permutations *}
  2953   {* simp rules and simprocs for analysing permutations *}
  2956 
  2954 
  2957 method_setup perm_simp_debug =
  2955 method_setup perm_simp_debug =
  2958   {* perm_eq_meth_debug *}
  2956   {* NominalPermeq.perm_eq_meth_debug *}
  2959   {* simp rules and simprocs for analysing permutations including debuging facilities *}
  2957   {* simp rules and simprocs for analysing permutations including debugging facilities *}
  2960 
  2958 
  2961 method_setup perm_full_simp =
  2959 method_setup perm_full_simp =
  2962   {* perm_full_eq_meth *}
  2960   {* NominalPermeq.perm_full_eq_meth *}
  2963   {* tactic for deciding equalities involving permutations *}
  2961   {* tactic for deciding equalities involving permutations *}
  2964 
  2962 
  2965 method_setup perm_full_simp_debug =
  2963 method_setup perm_full_simp_debug =
  2966   {* perm_full_eq_meth_debug *}
  2964   {* NominalPermeq.perm_full_eq_meth_debug *}
  2967   {* tactic for deciding equalities involving permutations including debuging facilities *}
  2965   {* tactic for deciding equalities involving permutations including debugging facilities *}
  2968 
  2966 
  2969 method_setup supports_simp =
  2967 method_setup supports_simp =
  2970   {* supports_meth *}
  2968   {* NominalPermeq.supports_meth *}
  2971   {* tactic for deciding whether something supports something else *}
  2969   {* tactic for deciding whether something supports something else *}
  2972 
  2970 
  2973 method_setup supports_simp_debug =
  2971 method_setup supports_simp_debug =
  2974   {* supports_meth_debug *}
  2972   {* NominalPermeq.supports_meth_debug *}
  2975   {* tactic for deciding whether something supports something else including debuging facilities *}
  2973   {* tactic for deciding whether something supports something else including debugging facilities *}
  2976 
  2974 
  2977 method_setup finite_guess =
  2975 method_setup finite_guess =
  2978   {* finite_gs_meth *}
  2976   {* NominalPermeq.finite_gs_meth *}
  2979   {* tactic for deciding whether something has finite support *}
  2977   {* tactic for deciding whether something has finite support *}
  2980 
  2978 
  2981 method_setup finite_guess_debug =
  2979 method_setup finite_guess_debug =
  2982   {* finite_gs_meth_debug *}
  2980   {* NominalPermeq.finite_gs_meth_debug *}
  2983   {* tactic for deciding whether something has finite support including debuging facilities *}
  2981   {* tactic for deciding whether something has finite support including debugging facilities *}
  2984 
  2982 
  2985 method_setup fresh_guess =
  2983 method_setup fresh_guess =
  2986   {* fresh_gs_meth *}
  2984   {* NominalPermeq.fresh_gs_meth *}
  2987   {* tactic for deciding whether an atom is fresh for something*}
  2985   {* tactic for deciding whether an atom is fresh for something*}
  2988 
  2986 
  2989 method_setup fresh_guess_debug =
  2987 method_setup fresh_guess_debug =
  2990   {* fresh_gs_meth_debug *}
  2988   {* NominalPermeq.fresh_gs_meth_debug *}
  2991   {* tactic for deciding whether an atom is fresh for something including debuging facilities *}
  2989   {* tactic for deciding whether an atom is fresh for something including debugging facilities *}
  2992 
  2990 
  2993 end
  2991 end