src/Sequents/simpdata.ML
changeset 46186 9ae331a1d8c5
parent 45659 09539cdffcd7
child 51717 9e7d1c139569
equal deleted inserted replaced
46185:afda84cd4d4b 46186:9ae331a1d8c5
    73   |> Simplifier.set_subgoaler asm_simp_tac
    73   |> Simplifier.set_subgoaler asm_simp_tac
    74   |> Simplifier.set_mksimps (K (map mk_meta_eq o atomize o gen_all))
    74   |> Simplifier.set_mksimps (K (map mk_meta_eq o atomize o gen_all))
    75   |> Simplifier.set_mkcong mk_meta_cong;
    75   |> Simplifier.set_mkcong mk_meta_cong;
    76 
    76 
    77 val LK_simps =
    77 val LK_simps =
    78    [triv_forall_equality, (* prunes params *)
    78    [@{thm triv_forall_equality}, (* prunes params *)
    79     @{thm refl} RS @{thm P_iff_T}] @
    79     @{thm refl} RS @{thm P_iff_T}] @
    80     @{thms conj_simps} @ @{thms disj_simps} @ @{thms not_simps} @
    80     @{thms conj_simps} @ @{thms disj_simps} @ @{thms not_simps} @
    81     @{thms imp_simps} @ @{thms iff_simps} @ @{thms quant_simps} @
    81     @{thms imp_simps} @ @{thms iff_simps} @ @{thms quant_simps} @
    82     @{thms all_simps} @ @{thms ex_simps} @
    82     @{thms all_simps} @ @{thms ex_simps} @
    83     [@{thm de_Morgan_conj}, @{thm de_Morgan_disj}, @{thm imp_disj1}, @{thm imp_disj2}] @
    83     [@{thm de_Morgan_conj}, @{thm de_Morgan_disj}, @{thm imp_disj1}, @{thm imp_disj2}] @