src/HOL/Proofs/Lambda/ListOrder.thy
changeset 67613 ce654b0e6d69
parent 61986 2461779da2b8
equal deleted inserted replaced
67610:4939494ed791 67613:ce654b0e6d69
    22   "step1 r =
    22   "step1 r =
    23     (\<lambda>ys xs. \<exists>us z z' vs. xs = us @ z # vs \<and> r z' z \<and> ys =
    23     (\<lambda>ys xs. \<exists>us z z' vs. xs = us @ z # vs \<and> r z' z \<and> ys =
    24       us @ z' # vs)"
    24       us @ z' # vs)"
    25 
    25 
    26 
    26 
    27 lemma step1_converse [simp]: "step1 (r^--1) = (step1 r)^--1"
    27 lemma step1_converse [simp]: "step1 (r\<inverse>\<inverse>) = (step1 r)\<inverse>\<inverse>"
    28   apply (unfold step1_def)
    28   apply (unfold step1_def)
    29   apply (blast intro!: order_antisym)
    29   apply (blast intro!: order_antisym)
    30   done
    30   done
    31 
    31 
    32 lemma in_step1_converse [iff]: "(step1 (r^--1) x y) = ((step1 r)^--1 x y)"
    32 lemma in_step1_converse [iff]: "(step1 (r\<inverse>\<inverse>) x y) = ((step1 r)\<inverse>\<inverse> x y)"
    33   apply auto
    33   apply auto
    34   done
    34   done
    35 
    35 
    36 lemma not_Nil_step1 [iff]: "\<not> step1 r [] xs"
    36 lemma not_Nil_step1 [iff]: "\<not> step1 r [] xs"
    37   apply (unfold step1_def)
    37   apply (unfold step1_def)