src/HOL/Bali/DefiniteAssignmentCorrect.thy
changeset 50710 32007a8db6bb
parent 44890 22f665a2e91c
child 51543 118f7cb0ee8e
equal deleted inserted replaced
50709:985c081a4f11 50710:32007a8db6bb
  1465       have "dom (locals (store s1)) \<subseteq> dom (locals (store s2))" 
  1465       have "dom (locals (store s1)) \<subseteq> dom (locals (store s2))" 
  1466         by simp
  1466         by simp
  1467       also
  1467       also
  1468       from ass_ok
  1468       from ass_ok
  1469       have "\<dots> \<subseteq> dom (locals (store (assign f v s2)))"
  1469       have "\<dots> \<subseteq> dom (locals (store (assign f v s2)))"
  1470         by (rule dom_locals_assign_mono)
  1470         by (rule dom_locals_assign_mono [where f = f])
  1471       finally show ?thesis by simp
  1471       finally show ?thesis by simp
  1472     next
  1472     next
  1473       case False
  1473       case False
  1474       with `G\<turnstile>s1 \<midarrow>e-\<succ>v\<rightarrow> s2`
  1474       with `G\<turnstile>s1 \<midarrow>e-\<succ>v\<rightarrow> s2`
  1475       have "s2=s1"
  1475       have "s2=s1"