src/HOL/Nominal/nominal_permeq.ML
changeset 55990 41c6b99c5fb7
parent 51717 9e7d1c139569
child 56230 3e449273942a
equal deleted inserted replaced
55989:55827fc7c0dd 55990:41c6b99c5fb7
   239       rtac (perm_fun_def RS meta_eq_to_obj_eq RS trans) i)
   239       rtac (perm_fun_def RS meta_eq_to_obj_eq RS trans) i)
   240 
   240 
   241 (* applies the ext-rule such that      *)
   241 (* applies the ext-rule such that      *)
   242 (*                                     *)
   242 (*                                     *)
   243 (*    f = g   goes to  /\x. f x = g x  *)
   243 (*    f = g   goes to  /\x. f x = g x  *)
   244 fun ext_fun_tac i = ("extensionality expansion of functions", rtac ext i);
   244 fun ext_fun_tac i = ("extensionality expansion of functions", rtac @{thm ext} i);
   245 
   245 
   246 
   246 
   247 (* perm_extend_simp_tac_i is perm_simp plus additional tactics        *)
   247 (* perm_extend_simp_tac_i is perm_simp plus additional tactics        *)
   248 (* to decide equation that come from support problems             *)
   248 (* to decide equation that come from support problems             *)
   249 (* since it contains looping rules the "recursion" - depth is set *)
   249 (* since it contains looping rules the "recursion" - depth is set *)