src/HOL/ATP.thy
changeset 39958 88c9aa5666de
parent 39951 ff60a6e4edfe
child 40121 e7a80c6752c9
equal deleted inserted replaced
39957:2f2d90cc31a2 39958:88c9aa5666de
     1 (*  Title:      HOL/ATP.thy
     1 (*  Title:      HOL/ATP.thy
     2     Author:     Fabian Immler, TU Muenchen
     2     Author:     Fabian Immler, TU Muenchen
     3     Author:     Jasmin Blanchette, TU Muenchen
     3     Author:     Jasmin Blanchette, TU Muenchen
     4 *)
     4 *)
     5 
     5 
     6 header {* Sledgehammer: Isabelle--ATP Linkup *}
     6 header {* Automatic Theorem Provers (ATPs) *}
     7 
     7 
     8 theory ATP
     8 theory ATP
     9 imports Plain
     9 imports Plain
    10 uses "Tools/ATP/atp_problem.ML"
    10 uses "Tools/ATP/atp_problem.ML"
    11      "Tools/ATP/atp_proof.ML"
    11      "Tools/ATP/atp_proof.ML"