krauss [Mon, 11 Feb 2008 15:40:21 +0100] rev 26056
Made theory names in ZF disjoint from HOL theory names to allow loading both developments
in a single session (but not merge them).
urbanc [Mon, 11 Feb 2008 15:19:17 +0100] rev 26055
tuned proofs and comments
wenzelm [Sun, 10 Feb 2008 20:49:48 +0100] rev 26054
tuned spaces;
wenzelm [Sun, 10 Feb 2008 20:49:47 +0100] rev 26053
tuned default position;
wenzelm [Sun, 10 Feb 2008 20:49:46 +0100] rev 26052
added default_properties;
wenzelm [Sun, 10 Feb 2008 20:49:45 +0100] rev 26051
added position_properties;
wenzelm [Sun, 10 Feb 2008 20:49:42 +0100] rev 26050
maintain default position;
wenzelm [Sat, 09 Feb 2008 12:56:12 +0100] rev 26049
overloading: reduced code redundancy, no xstrings here;
wenzelm [Sat, 09 Feb 2008 12:56:10 +0100] rev 26048
overloading: tuned signature;
berghofe [Thu, 07 Feb 2008 14:39:19 +0100] rev 26047
Instead of raising an exception, pred_set_conv now ignores conversion
rules that would cause a clash. This allows multiple interpretations
of locales containing inductive sets.
huffman [Thu, 07 Feb 2008 03:30:32 +0100] rev 26046
fix broken syntax translations
huffman [Wed, 06 Feb 2008 22:10:29 +0100] rev 26045
use ML antiquotations
krauss [Wed, 06 Feb 2008 16:06:40 +0100] rev 26044
lemma wf_union_compatible: "wf R ==> wf S ==> S O R <= R ==> wf (R Un S)"
chaieb [Wed, 06 Feb 2008 12:51:23 +0100] rev 26043
between constant removed
haftmann [Wed, 06 Feb 2008 08:34:51 +0100] rev 26042
continued