src/FOL/FOL.thy
changeset 41310 65631ca437c9
parent 36866 426d5781bb25
child 41779 a68f503805ed
equal deleted inserted replaced
41309:2e9bf718a7a1 41310:65631ca437c9
   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 eq}
   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
   389 *}
   389 *}
   390 
   390 
   391 setup Induct.setup
   391 setup Induct.setup
   392 declare case_split [cases type: o]
   392 declare case_split [cases type: o]
   393 
   393 
       
   394 
       
   395 hide_const (open) eq
       
   396 
   394 end
   397 end