Dear all,

please keep in mind that we are on track to (re-)introduce a type
constructor for sets.  I ask for solidarity: take this into account when
writing type annotations:

http://isabelle.in.tum.de/reports/Isabelle/file/2dd44cd8f963/src/HOL/Transitive_Closure.thy#l781

This should read:

lemma rel_pow_empty:
  "0 < n \<Longrightarrow> ({} :: ('a \<times> 'a) set) ^^ n = {}"
  by (cases n) auto

Violating this produces duplicated effort for backporting changes etc.,
which can be invested better.

        Florian

-- 

Home:
http://www.in.tum.de/~haftmann

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