src/CCL/CCL.thy
changeset 59755 f8d164ab0dc1
parent 59499 14095f771781
child 59763 56d2c357e6b5
equal deleted inserted replaced
59754:696d87036f04 59755:f8d164ab0dc1
   473   apply (rule EQgen_mono | assumption)+
   473   apply (rule EQgen_mono | assumption)+
   474   done
   474   done
   475 
   475 
   476 method_setup eq_coinduct3 = {*
   476 method_setup eq_coinduct3 = {*
   477   Scan.lift Args.name_inner_syntax >> (fn s => fn ctxt =>
   477   Scan.lift Args.name_inner_syntax >> (fn s => fn ctxt =>
   478     SIMPLE_METHOD' (res_inst_tac ctxt [(("R", 0), s)] @{thm eq_coinduct3}))
   478     SIMPLE_METHOD' (res_inst_tac ctxt [((("R", 0), Position.none), s)] @{thm eq_coinduct3}))
   479 *}
   479 *}
   480 
   480 
   481 
   481 
   482 subsection {* Untyped Case Analysis and Other Facts *}
   482 subsection {* Untyped Case Analysis and Other Facts *}
   483 
   483