wenzelm [Mon, 11 Feb 2008 21:32:13 +0100] rev 26060
imports Main;
wenzelm [Mon, 11 Feb 2008 21:32:12 +0100] rev 26059
removed unnecessary theory qualifiers;
wenzelm [Mon, 11 Feb 2008 21:32:11 +0100] rev 26058
simultaneous use_thys;
wenzelm [Mon, 11 Feb 2008 21:32:10 +0100] rev 26057
added Id;
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
haftmann [Wed, 06 Feb 2008 08:34:32 +0100] rev 26041
locales ACf, ACIf, ACIfSL and ACIfSLlin have been abandoned in favour of the existing algebraic classes ab_semigroup_mult, ab_semigroup_idem_mult, lower_semilattice (resp. uper_semilattice) and linorder
chaieb [Mon, 04 Feb 2008 17:00:01 +0100] rev 26040
replaced class by locale
wenzelm [Mon, 04 Feb 2008 12:13:08 +0100] rev 26039
*** MESSAGE REFERS TO 1.29 and 1.44 ***
sort_of_term: be permissive about _class *output* markers, to allow print translations invoke this function as well;
haftmann [Mon, 04 Feb 2008 10:52:40 +0100] rev 26038
towards quickcheck
haftmann [Mon, 04 Feb 2008 10:52:39 +0100] rev 26037
suppport for messages and indices
haftmann [Mon, 04 Feb 2008 10:52:37 +0100] rev 26036
added indexT
huffman [Sat, 02 Feb 2008 03:28:36 +0100] rev 26035
instance "*" :: (sq_ord, sq_ord) sq_ord
huffman [Sat, 02 Feb 2008 03:26:40 +0100] rev 26034
cleaned up
nipkow [Fri, 01 Feb 2008 18:01:06 +0100] rev 26033
modified MCollect syntax
haftmann [Fri, 01 Feb 2008 08:35:58 +0100] rev 26032
<TERM> syntax
haftmann [Fri, 01 Feb 2008 08:32:26 +0100] rev 26031
fixed term_of_sort
haftmann [Fri, 01 Feb 2008 08:32:10 +0100] rev 26030
fixed record problem
huffman [Fri, 01 Feb 2008 02:38:41 +0100] rev 26029
add lemmas prod_lessI and Pair_less_iff [simp]
huffman [Thu, 31 Jan 2008 22:00:31 +0100] rev 26028
add lemma is_lub_lambda
huffman [Thu, 31 Jan 2008 21:48:14 +0100] rev 26027
add lemma cpo_lubI
huffman [Thu, 31 Jan 2008 21:37:20 +0100] rev 26026
add lemma cpo_lubI
huffman [Thu, 31 Jan 2008 21:23:14 +0100] rev 26025
instances for class discrete_cpo
huffman [Thu, 31 Jan 2008 21:22:03 +0100] rev 26024
new lemma cont_discrete_cpo
huffman [Thu, 31 Jan 2008 21:21:22 +0100] rev 26023
new discrete_cpo axclass
haftmann [Thu, 31 Jan 2008 11:47:12 +0100] rev 26022
temporary adjustions
haftmann [Thu, 31 Jan 2008 11:44:46 +0100] rev 26021
explicit del_funcs
haftmann [Thu, 31 Jan 2008 11:44:43 +0100] rev 26020
proper term_of functions
haftmann [Thu, 31 Jan 2008 09:16:01 +0100] rev 26019
avoiding dynamic simpset lookup
huffman [Thu, 31 Jan 2008 01:31:19 +0100] rev 26018
new lemma is_lub_Pair; cleaned up some proofs
nipkow [Wed, 30 Jan 2008 17:36:03 +0100] rev 26017
commented stuff out
nipkow [Wed, 30 Jan 2008 17:34:21 +0100] rev 26016
added multiset comprehension
haftmann [Wed, 30 Jan 2008 10:57:47 +0100] rev 26015
idempotent semigroups
haftmann [Wed, 30 Jan 2008 10:57:46 +0100] rev 26014
dual orders and dual lattices
haftmann [Wed, 30 Jan 2008 10:57:44 +0100] rev 26013
Theorem Inductive.lfp_ordinal_induct generalized to complete lattices
huffman [Tue, 29 Jan 2008 18:00:12 +0100] rev 26012
new term-building combinators
haftmann [Tue, 29 Jan 2008 10:20:00 +0100] rev 26011
cleaned up evaluation interfaces
haftmann [Tue, 29 Jan 2008 10:19:58 +0100] rev 26010
tuned names
haftmann [Tue, 29 Jan 2008 10:19:56 +0100] rev 26009
treating division by zero properly
wenzelm [Mon, 28 Jan 2008 22:27:29 +0100] rev 26008
eliminated escaped white space;
wenzelm [Mon, 28 Jan 2008 22:27:27 +0100] rev 26007
basic scanners: produce symbol list instead of imploded string;
tuned signature;
wenzelm [Mon, 28 Jan 2008 22:27:27 +0100] rev 26006
* Outer syntax: string tokens no longer admit escaped white space;
wenzelm [Mon, 28 Jan 2008 22:27:26 +0100] rev 26005
location_of_position: Position.column_of (which counts Isabelle symbols, not characters);