src/FOL/FOL.thy
changeset 42802 51d7e74f6899
parent 42799 4e33894aec6d
child 42814 5af15f1e2ef6
equal deleted inserted replaced
42801:da4ad5f98953 42802:51d7e74f6899
   199 
   199 
   200 ML {*
   200 ML {*
   201   structure Blast = Blast
   201   structure Blast = Blast
   202   (
   202   (
   203     structure Classical = Cla
   203     structure Classical = Cla
   204     val thy = @{theory}
   204     val Trueprop_const = dest_Const @{const Trueprop}
   205     val equality_name = @{const_name eq}
   205     val equality_name = @{const_name eq}
   206     val not_name = @{const_name Not}
   206     val not_name = @{const_name Not}
   207     val notE = @{thm notE}
   207     val notE = @{thm notE}
   208     val ccontr = @{thm ccontr}
   208     val ccontr = @{thm ccontr}
   209     val hyp_subst_tac = Hypsubst.blast_hyp_subst_tac
   209     val hyp_subst_tac = Hypsubst.blast_hyp_subst_tac