src/HOL/Bali/Decl.thy
changeset 13601 fd3e3d6b37b2
parent 12937 0c4fd7529467
child 13688 a0b16d42d489
equal deleted inserted replaced
13600:9702c8636a7b 13601:fd3e3d6b37b2
    79   thus "x = y"
    79   thus "x = y"
    80   proof -
    80   proof -
    81     have "\<forall> x y. x < (y::acc_modi) \<and> y < x \<longrightarrow> False"
    81     have "\<forall> x y. x < (y::acc_modi) \<and> y < x \<longrightarrow> False"
    82       by (auto simp add: less_acc_def split add: acc_modi.split)
    82       by (auto simp add: less_acc_def split add: acc_modi.split)
    83     with prems show ?thesis
    83     with prems show ?thesis
    84       by  (auto simp add: le_acc_def)
    84       by (unfold le_acc_def) rules
    85   qed
    85   qed
    86   next
    86   next
    87   show "(x < y) = (x \<le> y \<and> x \<noteq> y)"
    87   show "(x < y) = (x \<le> y \<and> x \<noteq> y)"
    88     by (auto simp add: le_acc_def less_acc_def split add: acc_modi.split) 
    88     by (auto simp add: le_acc_def less_acc_def split add: acc_modi.split) 
    89   }
    89   }