# HG changeset patch # User haftmann # Date 1266402107 -3600 # Node ID 8e3b8b5f1e960ce61cbc2292e321b1c333c98435 # Parent 2e0966d6f951fdaf2d314dd69ad6ac0dea98330f example for executable choice diff -r 2e0966d6f951 -r 8e3b8b5f1e96 src/HOL/ex/Execute_Choice.thy --- a/src/HOL/ex/Execute_Choice.thy Wed Feb 17 10:43:20 2010 +0100 +++ b/src/HOL/ex/Execute_Choice.thy Wed Feb 17 11:21:47 2010 +0100 @@ -6,9 +6,18 @@ imports Main AssocList begin -definition valuesum :: "('a, 'b :: comm_monoid_add) mapping \ 'b" where +text {* + A trivial example: +*} + +definition valuesum :: "('a, 'b :: ab_group_add) mapping \ 'b" where "valuesum m = (\k \ Mapping.keys m. the (Mapping.lookup m k))" +text {* + Not that instead of defining @{term valuesum} with choice, we define it + directly and derive a description involving choice afterwards: +*} + lemma valuesum_rec: assumes fin: "finite (dom (Mapping.lookup m))" shows "valuesum m = (if Mapping.is_empty m then 0 else @@ -35,30 +44,59 @@ then show ?thesis by (simp add: keys_def valuesum_def is_empty_def) qed +text {* + In the context of the else-branch we can show that the exact choice is + irrelvant; in practice, finding this point where choice becomes irrelevant is the + most difficult thing! +*} + +lemma valuesum_choice: + "finite (Mapping.keys M) \ x \ Mapping.keys M \ y \ Mapping.keys M \ + the (Mapping.lookup M x) + valuesum (Mapping.delete x M) = + the (Mapping.lookup M y) + valuesum (Mapping.delete y M)" + by (simp add: valuesum_def keys_def setsum_diff) + +text {* + Given @{text valuesum_rec} as initial description, we stepwise refine it to something executable; + first, we formally insert the constructor @{term AList} and split the one equation into two, + where the second one provides the necessary context: +*} + lemma valuesum_rec_AList: - "valuesum (AList []) = 0" - "valuesum (AList (x # xs)) = (let l = (SOME l. l \ Mapping.keys (AList (x # xs))) in + shows [code]: "valuesum (AList []) = 0" + and "valuesum (AList (x # xs)) = (let l = (SOME l. l \ Mapping.keys (AList (x # xs))) in the (Mapping.lookup (AList (x # xs)) l) + valuesum (Mapping.delete l (AList (x # xs))))" by (simp_all add: valuesum_rec finite_dom_map_of is_empty_AList) -axioms - FIXME: "x \ A \ y \ A \ C x = C y" +text {* + As a side effect the precondition disappears (but note this has nothing to do with choice!). + The first equation deals with the uncritical empty case and can already be used for code generation. -lemma aux: "(SOME l. l \ Mapping.keys (AList (x # xs))) = fst (hd (x # xs))" -proof (rule FIXME) - show "fst (hd (x # xs)) \ Mapping.keys (AList (x # xs))" - by (simp add: keys_AList) - show "(SOME l. l \ Mapping.keys (AList (x # xs))) \ Mapping.keys (AList (x # xs))" - apply (rule someI) apply (simp add: keys_AList) apply auto - done -qed + Using @{text valuesum_choice}, we are able to prove an executable version of @{term valuesum}: +*} lemma valuesum_rec_exec [code]: - "valuesum (AList []) = 0" "valuesum (AList (x # xs)) = (let l = fst (hd (x # xs)) in the (Mapping.lookup (AList (x # xs)) l) + valuesum (Mapping.delete l (AList (x # xs))))" - by (simp_all add: valuesum_rec_AList aux) +proof - + let ?M = "AList (x # xs)" + let ?l1 = "(SOME l. l \ Mapping.keys ?M)" + let ?l2 = "fst (hd (x # xs))" + have "finite (Mapping.keys ?M)" by (simp add: keys_AList) + moreover have "?l1 \ Mapping.keys ?M" + by (rule someI) (auto simp add: keys_AList) + moreover have "?l2 \ Mapping.keys ?M" + by (simp add: keys_AList) + ultimately have "the (Mapping.lookup ?M ?l1) + valuesum (Mapping.delete ?l1 ?M) = + the (Mapping.lookup ?M ?l2) + valuesum (Mapping.delete ?l2 ?M)" + by (rule valuesum_choice) + then show ?thesis by (simp add: valuesum_rec_AList) +qed + +text {* + See how it works: +*} -value "valuesum (AList [(''abc'', (42::nat)), (''def'', 1705)])" +value "valuesum (AList [(''abc'', (42::int)), (''def'', 1705)])" end