src/HOL/HOL.thy
changeset 32176 893614e2c35c
parent 32172 c4e55f30d527
child 32402 5731300da417
equal deleted inserted replaced
32175:a89979440d2c 32176:893614e2c35c
   908 apply (tactic {* etac (Classical.dup_elim @{thm allE}) 1 *})
   908 apply (tactic {* etac (Classical.dup_elim @{thm allE}) 1 *})
   909 apply iprover
   909 apply iprover
   910 done
   910 done
   911 
   911 
   912 ML {*
   912 ML {*
   913 structure Blast = BlastFun
   913 structure Blast = Blast
   914 (
   914 (
       
   915   val thy = @{theory}
   915   type claset = Classical.claset
   916   type claset = Classical.claset
   916   val equality_name = @{const_name "op ="}
   917   val equality_name = @{const_name "op ="}
   917   val not_name = @{const_name Not}
   918   val not_name = @{const_name Not}
   918   val notE = @{thm notE}
   919   val notE = @{thm notE}
   919   val ccontr = @{thm ccontr}
   920   val ccontr = @{thm ccontr}