lh-l4v/lib/AutoLevity_Test.thy

55 lines
790 B
Plaintext
Raw Normal View History

2016-06-08 05:49:08 +00:00
(*
* 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)
2017-07-12 05:13:51 +00:00
*
2016-06-08 05:49:08 +00:00
*)
theory AutoLevity_Test
imports AutoLevity_Base AutoLevity_Hooks
begin
locale foo = fixes z assumes Z:"z" begin
ML \<open>Method.finish_text\<close>
2017-07-12 05:13:51 +00:00
lemma
X:
"(z \<and> z) \<and> (z \<and> z)"
apply (insert mp) apply (insert conjE)
apply (rule conjI)
subgoal
2017-07-12 05:13:51 +00:00
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"
2017-07-12 05:13:51 +00:00
apply
(rule
Z)
2017-07-12 05:13:51 +00:00
done
qed
done
end
interpretation foo "True" by (unfold_locales;
simp)
2017-07-12 05:13:51 +00:00
2016-06-08 05:49:08 +00:00
end