In rev. 544764f4324d

theory Foo
imports Main
begin

lemma less_dvd_minus:
  fixes m n :: nat
  assumes "m < n"
  shows "m dvd n ⟷ m dvd (n - m)"
  using assms apply arith oops

        Florian

-- 

PGP available:
http://home.informatik.tu-muenchen.de/haftmann/pgp/florian_haftmann_at_informatik_tu_muenchen_de

Attachment: signature.asc
Description: OpenPGP digital signature

_______________________________________________
isabelle-dev mailing list
isabelle-...@in.tum.de
https://mailmanbroy.informatik.tu-muenchen.de/mailman/listinfo/isabelle-dev

Reply via email to