Attribute for adjusting preconds.

Should work for corres-like rules. Works on an example. Needs
real testing.
This commit is contained in:
Thomas Sewell 2017-08-02 15:19:54 +10:00
parent eca624104c
commit 9f8297adc8
1 changed files with 163 additions and 0 deletions

View File

@ -0,0 +1,163 @@
(*
*
* Copyright 2017, Data61, CSIRO
*
* 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(DATA61_BSD)
*)
theory Corres_Adjust_Preconds
imports
"Corres_UL"
begin
text {*
Gadget for adjusting preconditions in a corres rule or similar.
Probably only useful for predicates with two or more related
preconditions, such as corres.
Used to do some_corres_rule[adj_corres some_intro_rule],
given e.g. some_intro_rule: @{prop "(s, t) \<in> sr \<Longrightarrow> P s \<Longrightarrow> Q t"}
Will apply this rule to solve @{prop "Q t"} components in either
precondition or any sub-conjunct, and will then try to put the
assumptions @{prop "P s"}, @{prop "(s, t) \<in> sr"} into the right
places. The premises of the rule can be in any given order.
Concrete example at the bottom.
*}
named_theorems corres_adjust_precond_structures
locale corres_adjust_preconds begin
definition
preconds :: "bool \<Rightarrow> bool \<Rightarrow> bool \<Rightarrow> bool \<Rightarrow> bool"
where
"preconds A B C D = (A \<and> B \<and> C \<and> D)"
definition
finalise_preconds :: "bool \<Rightarrow> bool"
where
"finalise_preconds A = True"
lemma consume_preconds:
"preconds A True True True \<Longrightarrow> A"
"preconds True B True True \<Longrightarrow> B"
"preconds True True C True \<Longrightarrow> C"
"preconds True True True D \<Longrightarrow> D"
by (simp_all add: preconds_def)
lemmas consume_preconds_True = consume_preconds(1)[where A=True]
lemma split_preconds_left:
"preconds (A \<and> A') (B \<and> B') (C \<and> C') (D \<and> D') \<Longrightarrow> preconds A B C D"
"preconds (A \<and> A') (B \<and> B') (C \<and> C') True \<Longrightarrow> preconds A B C True"
"preconds (A \<and> A') (B \<and> B') True True \<Longrightarrow> preconds A B True True"
"preconds (A \<and> A') True True True \<Longrightarrow> preconds A True True True"
by (simp_all add: preconds_def)
lemma split_preconds_right:
"preconds (A \<and> A') (B \<and> B') (C \<and> C') (D \<and> D') \<Longrightarrow> preconds A' B' C' D'"
"preconds (A \<and> A') (B \<and> B') (C \<and> C') True \<Longrightarrow> preconds A' B' C' True"
"preconds (A \<and> A') (B \<and> B') True True \<Longrightarrow> preconds A' B' True True"
"preconds (A \<and> A') True True True \<Longrightarrow> preconds A' True True True"
by (simp_all add: preconds_def)
lemma preconds_madness:
"preconds A B C D \<Longrightarrow> (preconds A B C D \<Longrightarrow> Q) \<Longrightarrow> finalise_preconds (A \<and> B \<and> C \<and> D) \<Longrightarrow> Q"
by simp
lemma finalise_preconds:
"finalise_preconds True"
"finalise_preconds A \<Longrightarrow> finalise_preconds B \<Longrightarrow> finalise_preconds (A \<and> B)"
"finalise_preconds X"
by (simp_all add: finalise_preconds_def)
lemma corres_adjust_pre:
"corres_underlying R nf nf' rs P Q f f'
\<Longrightarrow> (\<And>s s'. (s, s') \<in> R \<Longrightarrow> preconds (P1 s) (Q1 s') True True \<Longrightarrow> P s)
\<Longrightarrow> (\<And>s s'. (s, s') \<in> R \<Longrightarrow> preconds (Q2 s') (P2 s) True True \<Longrightarrow> Q s')
\<Longrightarrow> corres_underlying R nf nf' rs (\<lambda>s. P1 s \<and> P2 s) (\<lambda>s'. Q1 s' \<and> Q2 s') f f'"
apply (erule stronger_corres_guard_imp)
apply (simp add: preconds_def)+
done
ML {*
structure Corres_Adjust_Preconds = struct
val def_intros = @{thms conjI pred_conj_app[THEN iffD2]
bipred_conj_app[THEN fun_cong, THEN iffD2]}
fun intro_split ctxt intros i =
((resolve_tac ctxt intros
THEN_ALL_NEW (TRY o assume_tac ctxt))
THEN_ALL_NEW (fn j => (EVERY (replicate (j - i) (dresolve_tac ctxt @{thms split_preconds_left} j)))
THEN dresolve_tac ctxt @{thms split_preconds_right} j)) i
fun handle_preconds ctxt intros =
TRY o (eresolve_tac ctxt [@{thm preconds_madness}]
THEN' REPEAT_ALL_NEW (eresolve_tac ctxt @{thms consume_preconds_True}
ORELSE' intro_split ctxt (intros @ def_intros)
ORELSE' eresolve_tac ctxt @{thms consume_preconds})
THEN' REPEAT_ALL_NEW (resolve_tac ctxt @{thms finalise_preconds})
)
fun mk_adj_preconds ctxt intros rule = let
val xs = [rule] RL (Named_Theorems.get ctxt @{named_theorems corres_adjust_precond_structures})
val x = case xs of
[] => raise THM ("no unifier with corres_adjust_precond_structures", 1, [rule])
| xs => hd xs
in x
|> ALLGOALS (handle_preconds ctxt intros)
|> Seq.hd
|> Simplifier.simplify (clear_simpset ctxt addsimps @{thms conj_assoc simp_thms(21-22)})
end
val setup =
Attrib.setup @{binding "adj_corres"}
((Attrib.thms -- Args.context)
>> (fn (intros, ctxt) => Thm.rule_attribute [] (K (mk_adj_preconds ctxt intros))))
"use argument theorems to adjust a corres theorem."
end
*}
end
declare corres_adjust_preconds.corres_adjust_pre[corres_adjust_precond_structures]
setup Corres_Adjust_Preconds.setup
experiment begin
definition
test_sr :: "(nat \<times> nat) set"
where
"test_sr = {(x, y). y = 2 * x}"
lemma test_corres:
"corres_underlying test_sr nf nf' dc (\<lambda>x. x < 40) (\<lambda>y. y < 30 \<and> y = 6)
(modify (\<lambda>x. x + 2)) (modify (\<lambda>y. 10))"
by (simp add: corres_underlying_def simpler_modify_def test_sr_def)
lemma test_adj_precond:
"(x, y) \<in> test_sr \<Longrightarrow> x = 3 \<Longrightarrow> y = 6"
by (simp add: test_sr_def)
ML {*
Corres_Adjust_Preconds.mk_adj_preconds @{context} [@{thm test_adj_precond}] @{thm test_corres}
*}
lemmas foo = test_corres test_corres[adj_corres test_adj_precond]
end
end