(* * Copyright 2014, NICTA * * This software may be distributed and modified according to the terms of * the BSD 2-Clause license. Note that NO WARRANTY is provided. * See "LICENSE_BSD2.txt" for details. * * @TAG(NICTA_BSD) * *) theory AutoLevity_Test imports AutoLevity_Base AutoLevity_Hooks begin locale foo = fixes z assumes Z:"z" begin ML \Method.finish_text\ lemma X: "(z \ z) \ (z \ z)" apply (insert mp) apply (insert conjE) apply (rule conjI) subgoal apply (rule conjI) by (rule Z) (rule Z) subgoal apply (rule conjI) subgoal subgoal subgoal apply (insert impE) by (rule Z) done done proof - show "z" apply (rule Z) done qed done end interpretation foo "True" by (unfold_locales; simp) end