src/HOL/Decision_Procs/Parametric_Ferrante_Rackoff.thy
changeset 54742 7a86358a3c0b
parent 54230 b1d955791529
child 55417 01fbfb60c33e
equal deleted inserted replaced
54741:010eefa0a4f3 54742:7a86358a3c0b
  2918 ML {* 
  2918 ML {* 
  2919 structure Parametric_Ferrante_Rackoff = 
  2919 structure Parametric_Ferrante_Rackoff = 
  2920 struct
  2920 struct
  2921 
  2921 
  2922 fun tactic ctxt alternative T ps = 
  2922 fun tactic ctxt alternative T ps = 
  2923   Object_Logic.full_atomize_tac
  2923   Object_Logic.full_atomize_tac ctxt
  2924   THEN' CSUBGOAL (fn (g, i) =>
  2924   THEN' CSUBGOAL (fn (g, i) =>
  2925     let
  2925     let
  2926       val th = frpar_oracle (ctxt, alternative, T, ps, g)
  2926       val th = frpar_oracle (ctxt, alternative, T, ps, g)
  2927     in rtac (th RS iffD2) i end);
  2927     in rtac (th RS iffD2) i end);
  2928 
  2928