Wed, 06 Feb 2008 16:06:40 +0100 krauss lemma wf_union_compatible: "wf R ==> wf S ==> S O R <= R ==> wf (R Un S)"
Wed, 06 Feb 2008 12:51:23 +0100 chaieb between constant removed
Wed, 06 Feb 2008 08:34:51 +0100 haftmann continued
Wed, 06 Feb 2008 08:34:32 +0100 haftmann 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
Mon, 04 Feb 2008 17:00:01 +0100 chaieb replaced class by locale
Mon, 04 Feb 2008 12:13:08 +0100 wenzelm *** MESSAGE REFERS TO 1.29 and 1.44 ***
Mon, 04 Feb 2008 10:52:40 +0100 haftmann towards quickcheck
Mon, 04 Feb 2008 10:52:39 +0100 haftmann suppport for messages and indices
Mon, 04 Feb 2008 10:52:37 +0100 haftmann added indexT
Sat, 02 Feb 2008 03:28:36 +0100 huffman instance "*" :: (sq_ord, sq_ord) sq_ord
Sat, 02 Feb 2008 03:26:40 +0100 huffman cleaned up
Fri, 01 Feb 2008 18:01:06 +0100 nipkow modified MCollect syntax
Fri, 01 Feb 2008 08:35:58 +0100 haftmann <TERM> syntax
Fri, 01 Feb 2008 08:32:26 +0100 haftmann fixed term_of_sort
Fri, 01 Feb 2008 08:32:10 +0100 haftmann fixed record problem
Fri, 01 Feb 2008 02:38:41 +0100 huffman add lemmas prod_lessI and Pair_less_iff [simp]
Thu, 31 Jan 2008 22:00:31 +0100 huffman add lemma is_lub_lambda
Thu, 31 Jan 2008 21:48:14 +0100 huffman add lemma cpo_lubI
Thu, 31 Jan 2008 21:37:20 +0100 huffman add lemma cpo_lubI
Thu, 31 Jan 2008 21:23:14 +0100 huffman instances for class discrete_cpo
Thu, 31 Jan 2008 21:22:03 +0100 huffman new lemma cont_discrete_cpo
Thu, 31 Jan 2008 21:21:22 +0100 huffman new discrete_cpo axclass
Thu, 31 Jan 2008 11:47:12 +0100 haftmann temporary adjustions
Thu, 31 Jan 2008 11:44:46 +0100 haftmann explicit del_funcs
Thu, 31 Jan 2008 11:44:43 +0100 haftmann proper term_of functions
Thu, 31 Jan 2008 09:16:01 +0100 haftmann avoiding dynamic simpset lookup
Thu, 31 Jan 2008 01:31:19 +0100 huffman new lemma is_lub_Pair; cleaned up some proofs
Wed, 30 Jan 2008 17:36:03 +0100 nipkow commented stuff out
Wed, 30 Jan 2008 17:34:21 +0100 nipkow added multiset comprehension
Wed, 30 Jan 2008 10:57:47 +0100 haftmann idempotent semigroups
Wed, 30 Jan 2008 10:57:46 +0100 haftmann dual orders and dual lattices
Wed, 30 Jan 2008 10:57:44 +0100 haftmann Theorem Inductive.lfp_ordinal_induct generalized to complete lattices
Tue, 29 Jan 2008 18:00:12 +0100 huffman new term-building combinators
Tue, 29 Jan 2008 10:20:00 +0100 haftmann cleaned up evaluation interfaces
Tue, 29 Jan 2008 10:19:58 +0100 haftmann tuned names
Tue, 29 Jan 2008 10:19:56 +0100 haftmann treating division by zero properly
Mon, 28 Jan 2008 22:27:29 +0100 wenzelm eliminated escaped white space;
Mon, 28 Jan 2008 22:27:27 +0100 wenzelm basic scanners: produce symbol list instead of imploded string;
Mon, 28 Jan 2008 22:27:27 +0100 wenzelm * Outer syntax: string tokens no longer admit escaped white space;
Mon, 28 Jan 2008 22:27:26 +0100 wenzelm location_of_position: Position.column_of (which counts Isabelle symbols, not characters);
Mon, 28 Jan 2008 22:27:24 +0100 wenzelm added count/counted: improved position handling for token syntax;
Mon, 28 Jan 2008 22:27:23 +0100 wenzelm added column field;
Mon, 28 Jan 2008 22:27:23 +0100 wenzelm T.count/counted: improved position handling for token syntax;
Mon, 28 Jan 2008 22:27:21 +0100 wenzelm added column property;
Mon, 28 Jan 2008 22:27:20 +0100 wenzelm removed redundant repeatd scanner combinator;
Mon, 28 Jan 2008 22:27:19 +0100 wenzelm added ::: / @@@ scanner combinators;
Mon, 28 Jan 2008 18:18:19 +0100 berghofe Tuned uniqueness proof for recursion combinator.
Mon, 28 Jan 2008 18:17:42 +0100 berghofe Cleaned up simproc code.
Mon, 28 Jan 2008 08:14:31 +0100 urbanc tuned the proof of the substitution lemma
Sun, 27 Jan 2008 22:21:39 +0100 wenzelm rename_client_map_tac: avoid ill-defined thm reference;
Sun, 27 Jan 2008 22:21:37 +0100 wenzelm use_thy: do not set implicit ML context anymore;
Sun, 27 Jan 2008 22:21:35 +0100 wenzelm added ambiguity_limit (restricts parse trees / terms printed in messages);
Sun, 27 Jan 2008 22:21:34 +0100 wenzelm renamed thms_containing_limit to FindTheorems.limit;
Sun, 27 Jan 2008 20:04:32 +0100 wenzelm eliminated some legacy ML files;
Sun, 27 Jan 2008 20:04:31 +0100 wenzelm added bind_thms;
Sun, 27 Jan 2008 20:04:30 +0100 wenzelm tuned;
Sun, 27 Jan 2008 18:32:32 +0100 wenzelm removed legacy ML file;
Sat, 26 Jan 2008 23:15:33 +0100 wenzelm syntax error: unified output of priorities;
Sat, 26 Jan 2008 22:14:07 +0100 wenzelm syntax error: reduced spam -- print expected nonterminals instead of terminals;
Sat, 26 Jan 2008 20:01:37 +0100 wenzelm avoid redundant escaping of Isabelle symbols;
(0) -10000 -3000 -1000 -300 -100 -60 +60 +100 +300 +1000 +3000 +10000 +30000 tip