Theory Prerequisites
theory Prerequisites
imports Main
keywords "lemmas_with" :: thy_decl
begin
context
fixes Rep Abs A T
assumes type: "type_definition Rep Abs A"
assumes T_def: "T ≡ (λ(x::'a) (y::'b). x = Rep y)"
begin
lemma type_definition_Domainp: "Domainp T = (λx. x ∈ A)"
proof -
interpret type_definition Rep Abs A by(rule type)
show ?thesis
unfolding Domainp_iff[abs_def] T_def fun_eq_iff
by (metis Abs_inverse Rep)
qed
end
subsection ‹setting up transfer for local typedef›
lemmas [transfer_rule] =
right_total_All_transfer
right_total_UNIV_transfer
right_total_Ex_transfer
locale local_typedef = fixes S ::"'b set" and s::"'s itself"
assumes Ex_type_definition_S: "∃(Rep::'s ⇒ 'b) (Abs::'b ⇒ 's). type_definition Rep Abs S"
begin
definition "rep = fst (SOME (Rep::'s ⇒ 'b, Abs). type_definition Rep Abs S)"
definition "Abs = snd (SOME (Rep::'s ⇒ 'b, Abs). type_definition Rep Abs S)"
lemma type_definition_S: "type_definition rep Abs S"
unfolding Abs_def rep_def split_beta'
by (rule someI_ex) (use Ex_type_definition_S in auto)
lemma rep_in_S[simp]: "rep x ∈ S"
and rep_inverse[simp]: "Abs (rep x) = x"
and Abs_inverse[simp]: "y ∈ S ⟹ rep (Abs y) = y"
using type_definition_S
unfolding type_definition_def by auto
definition cr_S where "cr_S ≡ λs b. s = rep b"
lemmas Domainp_cr_S = type_definition_Domainp[OF type_definition_S cr_S_def, transfer_domain_rule]
lemmas right_total_cr_S = typedef_right_total[OF type_definition_S cr_S_def, transfer_rule]
and bi_unique_cr_S = typedef_bi_unique[OF type_definition_S cr_S_def, transfer_rule]
and left_unique_cr_S = typedef_left_unique[OF type_definition_S cr_S_def, transfer_rule]
and right_unique_cr_S = typedef_right_unique[OF type_definition_S cr_S_def, transfer_rule]
lemma cr_S_rep[intro, simp]: "cr_S (rep a) a" by (simp add: cr_S_def)
lemma cr_S_Abs[intro, simp]: "a∈S ⟹ cr_S a (Abs a)" by (simp add: cr_S_def)
end
subsection ‹some ›
subsection ‹Tool support›
lemmas subset_iff' = subset_iff[folded Ball_def]
ML ‹
structure More_Simplifier =
struct
fun asm_full_var_simplify ctxt thm =
let
val ((_, [thm']), ctxt') = Variable.import false [thm] ctxt
in
Simplifier.asm_full_simplify ctxt' thm'
|> singleton (Variable.export ctxt' ctxt)
|> Drule.zero_var_indexes
end
fun var_simplify_only ctxt ths thm =
asm_full_var_simplify (Raw_Simplifier.clear_simpset ctxt addsimps ths) thm
val var_simplified = Attrib.thms >>
(fn ths => Thm.rule_attribute ths
(fn context => var_simplify_only (Context.proof_of context) ths))
val _ = Theory.setup (Attrib.setup \<^binding>‹var_simplified› var_simplified "simplified rule (with vars)")
end
›
ML ‹
val _ = Outer_Syntax.local_theory' \<^command_keyword>‹lemmas_with› "note theorems with (the same) attributes"
(Parse.attribs --| \<^keyword>‹:› -- Parse_Spec.name_facts -- Parse.for_fixes
>> (fn (((attrs),facts), fixes) =>
#2 oo Specification.theorems_cmd Thm.theoremK
(map (apsnd (map (apsnd (fn xs => attrs@xs)))) facts) fixes))
›
end