src/HOL/HOL.thy
changeset 58963 26bf09b95dda
parent 58958 114255dce178
child 59028 df7476e79558
equal deleted inserted replaced
58960:4bee6d8c1500 58963:26bf09b95dda
  1980       | wrong_prem (Bound _) = true
  1980       | wrong_prem (Bound _) = true
  1981       | wrong_prem _ = false;
  1981       | wrong_prem _ = false;
  1982     val filter_right = filter (not o wrong_prem o HOLogic.dest_Trueprop o hd o Thm.prems_of);
  1982     val filter_right = filter (not o wrong_prem o HOLogic.dest_Trueprop o hd o Thm.prems_of);
  1983   in
  1983   in
  1984     fun smp i = funpow i (fn m => filter_right ([spec] RL m)) ([mp]);
  1984     fun smp i = funpow i (fn m => filter_right ([spec] RL m)) ([mp]);
  1985     fun smp_tac j = EVERY'[dresolve_tac (smp j), assume_tac];
  1985     fun smp_tac ctxt j = EVERY'[dresolve_tac (smp j), assume_tac ctxt];
  1986   end;
  1986   end;
  1987 
  1987 
  1988   local
  1988   local
  1989     val nnf_ss =
  1989     val nnf_ss =
  1990       simpset_of (put_simpset HOL_basic_ss @{context} addsimps @{thms simp_thms nnf_simps});
  1990       simpset_of (put_simpset HOL_basic_ss @{context} addsimps @{thms simp_thms nnf_simps});