src/HOL/Try0.thy
author wenzelm
Tue, 12 Aug 2025 11:19:08 +0200
changeset 82996 4a77ce6d4e07
parent 82363 3a7fc54b50ca
permissions -rw-r--r--
obsolete (see 5d562dd387ae);

(* Title:      HOL/Try0.thy
   Author:     Jasmin Blanchette, LMU Muenchen
   Author:     Martin Desharnais, LMU Muenchen
   Author:     Fabian Huch, TU Muenchen
*)

theory Try0
  imports Pure
  keywords "try0" :: diag
begin

ML_file \<open>Tools/try0.ML\<close>
ML_file \<open>Tools/try0_util.ML\<close>

ML \<open>
val () =
  Try0.register_proof_method "simp" {run_if_auto_try = true}
    (Try0_Util.apply_raw_named_method "simp" false Try0_Util.simp_attrs Simplifier_Trace.disable)
  handle Symtab.DUP _ => ()
\<close>

end