src/FOL/FOL.thy
changeset 32960 69916a850301
parent 32261 05e687ddbcee
child 34914 e391c3de0f6b
equal deleted inserted replaced
32959:23a8c5ac35f8 32960:69916a850301
   172 
   172 
   173 ML {*
   173 ML {*
   174   structure Blast = Blast
   174   structure Blast = Blast
   175   (
   175   (
   176     val thy = @{theory}
   176     val thy = @{theory}
   177     type claset	= Cla.claset
   177     type claset = Cla.claset
   178     val equality_name = @{const_name "op ="}
   178     val equality_name = @{const_name "op ="}
   179     val not_name = @{const_name Not}
   179     val not_name = @{const_name Not}
   180     val notE	= @{thm notE}
   180     val notE = @{thm notE}
   181     val ccontr	= @{thm ccontr}
   181     val ccontr = @{thm ccontr}
   182     val contr_tac = Cla.contr_tac
   182     val contr_tac = Cla.contr_tac
   183     val dup_intr	= Cla.dup_intr
   183     val dup_intr = Cla.dup_intr
   184     val hyp_subst_tac = Hypsubst.blast_hyp_subst_tac
   184     val hyp_subst_tac = Hypsubst.blast_hyp_subst_tac
   185     val rep_cs = Cla.rep_cs
   185     val rep_cs = Cla.rep_cs
   186     val cla_modifiers = Cla.cla_modifiers
   186     val cla_modifiers = Cla.cla_modifiers
   187     val cla_meth' = Cla.cla_meth'
   187     val cla_meth' = Cla.cla_meth'
   188   );
   188   );