src/HOL/HOL.thy
changeset 51304 0e71a248cacb
parent 51021 1cf4faed8b22
child 51314 eac4bb5adbf9
equal deleted inserted replaced
51303:4cca272150ab 51304:0e71a248cacb
  1985 
  1985 
  1986 
  1986 
  1987 subsection {* Legacy tactics and ML bindings *}
  1987 subsection {* Legacy tactics and ML bindings *}
  1988 
  1988 
  1989 ML {*
  1989 ML {*
  1990 fun strip_tac i = REPEAT (resolve_tac [impI, allI] i);
       
  1991 
       
  1992 (* combination of (spec RS spec RS ...(j times) ... spec RS mp) *)
  1990 (* combination of (spec RS spec RS ...(j times) ... spec RS mp) *)
  1993 local
  1991 local
  1994   fun wrong_prem (Const (@{const_name All}, _) $ Abs (_, _, t)) = wrong_prem t
  1992   fun wrong_prem (Const (@{const_name All}, _) $ Abs (_, _, t)) = wrong_prem t
  1995     | wrong_prem (Bound _) = true
  1993     | wrong_prem (Bound _) = true
  1996     | wrong_prem _ = false;
  1994     | wrong_prem _ = false;