src/HOL/Bali/Decl.thy
changeset 17589 58eeffd73be1
parent 16417 9bc16273c2d4
child 17778 93d7e524417a
equal deleted inserted replaced
17588:f2bd501398ee 17589:58eeffd73be1
    78   thus "x = y"
    78   thus "x = y"
    79   proof -
    79   proof -
    80     have "\<forall> x y. x < (y::acc_modi) \<and> y < x \<longrightarrow> False"
    80     have "\<forall> x y. x < (y::acc_modi) \<and> y < x \<longrightarrow> False"
    81       by (auto simp add: less_acc_def split add: acc_modi.split)
    81       by (auto simp add: less_acc_def split add: acc_modi.split)
    82     with prems show ?thesis
    82     with prems show ?thesis
    83       by (unfold le_acc_def) rules
    83       by (unfold le_acc_def) iprover
    84   qed
    84   qed
    85   next
    85   next
    86   show "(x < y) = (x \<le> y \<and> x \<noteq> y)"
    86   show "(x < y) = (x \<le> y \<and> x \<noteq> y)"
    87     by (auto simp add: le_acc_def less_acc_def split add: acc_modi.split) 
    87     by (auto simp add: le_acc_def less_acc_def split add: acc_modi.split) 
    88   }
    88   }