src/HOL/Library/Nested_Environment.thy
changeset 18576 8d98b7711e47
parent 18447 da548623916a
child 20503 503ac4c5ef91
equal deleted inserted replaced
18575:9ccfd1d1e874 18576:8d98b7711e47
   191   shows "\<exists>e. lookup env xs = Some e"
   191   shows "\<exists>e. lookup env xs = Some e"
   192 proof -
   192 proof -
   193   from prems have "lookup env (xs @ ys) \<noteq> None" by simp
   193   from prems have "lookup env (xs @ ys) \<noteq> None" by simp
   194   then have "lookup env xs \<noteq> None"
   194   then have "lookup env xs \<noteq> None"
   195     by (rule contrapos_nn) (simp only: lookup_append_none)
   195     by (rule contrapos_nn) (simp only: lookup_append_none)
   196   then show ?thesis by (simp add: not_None_eq)
   196   then show ?thesis by (simp)
   197 qed
   197 qed
   198 
   198 
   199 text {*
   199 text {*
   200   The subsequent statement describes in more detail how a successful
   200   The subsequent statement describes in more detail how a successful
   201   @{term lookup} with a non-empty path results in a certain situation
   201   @{term lookup} with a non-empty path results in a certain situation