Fri, 15 Aug 2008 15:50:52 +0200 wenzelm renamed T.source_of' to T.source_position_of;
Fri, 15 Aug 2008 15:50:50 +0200 wenzelm output_markup: check Markup.is_none;
Fri, 15 Aug 2008 15:50:49 +0200 wenzelm added is_none;
Fri, 15 Aug 2008 15:50:44 +0200 wenzelm Args.name_source(_position) for proper position information;
Thu, 14 Aug 2008 21:06:07 +0200 wenzelm [source=false] for quoted antiquotation avoids quote-escapes in output;
Thu, 14 Aug 2008 20:29:38 +0200 wenzelm report antiquotations;
Thu, 14 Aug 2008 20:29:37 +0200 wenzelm tuned;
Thu, 14 Aug 2008 20:13:43 +0200 wenzelm report ML_source;
Thu, 14 Aug 2008 20:13:42 +0200 wenzelm renamed P.ml_source to P.ML_source;
Thu, 14 Aug 2008 20:13:41 +0200 wenzelm report doc_source;
Thu, 14 Aug 2008 20:13:40 +0200 wenzelm added ML_source, doc_source;
Thu, 14 Aug 2008 19:52:40 +0200 wenzelm antiquotes: proper SymbolPos decoding, adapted Antiquote.read/Antiq;
Thu, 14 Aug 2008 19:52:39 +0200 wenzelm added source_of';
Thu, 14 Aug 2008 19:52:37 +0200 wenzelm P.doc_source and P.ml_sorce for proper SymbolPos.text;
Thu, 14 Aug 2008 19:52:36 +0200 wenzelm oracle, header/local_theory/proof_markup: pass SymbolPos.text;
Thu, 14 Aug 2008 19:52:35 +0200 wenzelm use SymbolPos.T list directly, instead of encoded SymbolPos.text;
Thu, 14 Aug 2008 16:52:56 +0200 wenzelm ML_Context.add_antiq: pass position;
Thu, 14 Aug 2008 16:52:54 +0200 wenzelm ML_Context.add_antiq: pass position;
Thu, 14 Aug 2008 16:52:52 +0200 wenzelm retrieve_thms: transfer fact position to result;
Thu, 14 Aug 2008 16:52:51 +0200 wenzelm moved basic thm operations from structure PureThy to Thm;
Thu, 14 Aug 2008 16:52:46 +0200 wenzelm moved basic thm operations from structure PureThy to Thm (cf. more_thm.ML);
Thu, 14 Aug 2008 11:55:05 +0200 wenzelm made SML/NJ happy;
Wed, 13 Aug 2008 20:57:40 +0200 wenzelm removed obsolete present_html -- now part of regular theory presentation;
Wed, 13 Aug 2008 20:57:39 +0200 wenzelm removed obsolete verbatim_source, results, chapter, section etc.;
Wed, 13 Aug 2008 20:57:37 +0200 wenzelm removed obsolete verbatim_source, results, chapter, section etc.;
Wed, 13 Aug 2008 20:57:35 +0200 wenzelm ProofDisplay.add_hook;
Wed, 13 Aug 2008 20:57:33 +0200 wenzelm simplified present_local_theory/proof;
Wed, 13 Aug 2008 20:57:33 +0200 wenzelm ProofDisplay.theory_results;
Wed, 13 Aug 2008 20:57:31 +0200 wenzelm removed obsolete present_results;
Wed, 13 Aug 2008 20:57:30 +0200 wenzelm scan: SymbolPos.tabify_content when creating tokens (for proper presentation output);
Wed, 13 Aug 2008 20:57:30 +0200 wenzelm load_thy: no untabify (preserve position information!), present spans instead of verbatim source;
Wed, 13 Aug 2008 20:57:28 +0200 wenzelm simplified markup commands;
Wed, 13 Aug 2008 20:57:26 +0200 wenzelm simplified markup commands -- removed obsolete Present.results, always check text;
Wed, 13 Aug 2008 20:57:24 +0200 wenzelm added untabify_content;
Wed, 13 Aug 2008 20:57:22 +0200 wenzelm tuned;
Wed, 13 Aug 2008 20:57:20 +0200 wenzelm removed obsolete untabify (superceded by SymbolPos.tabify_content);
Wed, 13 Aug 2008 20:57:18 +0200 wenzelm tuned document;
Wed, 13 Aug 2008 20:57:16 +0200 wenzelm removed obsolete theorems;
Wed, 13 Aug 2008 03:00:33 +0200 berghofe Changed proof of strong induction rule to avoid infinite loop
Tue, 12 Aug 2008 21:48:59 +0200 wenzelm token_kind_markup: complete coverage;
Tue, 12 Aug 2008 21:28:09 +0200 wenzelm OuterSyntax.scan: pass position;
Tue, 12 Aug 2008 21:28:07 +0200 wenzelm message: ignored if body empty;
Tue, 12 Aug 2008 21:28:05 +0200 wenzelm load_thy: removed obsolete dir argument;
Tue, 12 Aug 2008 21:28:03 +0200 wenzelm abstract type span, tuned interfaces;
Tue, 12 Aug 2008 21:28:01 +0200 wenzelm adapted ThyEdit operations;
Tue, 12 Aug 2008 21:27:59 +0200 wenzelm added ignored, malformed transitions;
Tue, 12 Aug 2008 21:27:57 +0200 wenzelm Symbol.source/OuterLex.source: more explicit do_recover argument;
Tue, 12 Aug 2008 21:27:55 +0200 wenzelm Isabelle.command: inline former OuterSyntax.prepare_command;
Tue, 12 Aug 2008 21:27:53 +0200 wenzelm load thy_edit.ML before outer_syntax.ML;
Tue, 12 Aug 2008 21:27:51 +0200 wenzelm renamed unknown_span to malformed_span;
Tue, 12 Aug 2008 21:27:48 +0200 wenzelm Symbol.source/OuterLex.source: more explicit do_recover argument;
Tue, 12 Aug 2008 21:27:46 +0200 wenzelm updated generated file;
Mon, 11 Aug 2008 22:25:45 +0200 haftmann rudimentary code setup for set operations
Mon, 11 Aug 2008 22:06:51 +0200 wenzelm <applet>: more XHTML 1.0 Transitional conformance;
Mon, 11 Aug 2008 22:06:49 +0200 wenzelm Isar.command: OuterSyntax.prepare_command_failsafe defers syntax errors until execution time;
Mon, 11 Aug 2008 20:56:32 +0200 wenzelm <pre>: removed xml:space, is already default;
Mon, 11 Aug 2008 18:37:51 +0200 wenzelm produce XHTML 1.0 Transitional;
Mon, 11 Aug 2008 18:37:49 +0200 wenzelm renamed Markup.class to Markup.tclass, to avoid potential conflicts with spacial meaning in markup languages (e.g. HTML);
Mon, 11 Aug 2008 17:37:48 +0200 wenzelm Isar.command: do not set position of enclosing transaction, to avoid of clash with the one being prepared here!
Mon, 11 Aug 2008 14:50:04 +0200 haftmann changed code setup
Mon, 11 Aug 2008 14:50:02 +0200 haftmann re-arranged class dense_linear_order
Mon, 11 Aug 2008 14:50:00 +0200 haftmann rudimentary code setup for set operations
Mon, 11 Aug 2008 14:49:53 +0200 haftmann moved class wellorder to theory Orderings
Sun, 10 Aug 2008 12:38:26 +0200 wenzelm added parse_token (from proof_context.ML);
Sun, 10 Aug 2008 12:38:25 +0200 wenzelm read_tyname/const/const_proper: report position;
Sun, 10 Aug 2008 12:38:24 +0200 wenzelm pass position to get_fact;
Sun, 10 Aug 2008 12:38:23 +0200 wenzelm pass token source to typ/term etc.;
Sun, 10 Aug 2008 12:38:22 +0200 wenzelm added name property operation;
Sat, 09 Aug 2008 22:43:59 +0200 wenzelm renamed ML_Lex.val_of to content_of;
Sat, 09 Aug 2008 22:43:58 +0200 wenzelm unified Args.T with OuterLex.token, renamed some operations;
Sat, 09 Aug 2008 22:43:57 +0200 wenzelm unified Args.T with OuterLex.token;
Sat, 09 Aug 2008 22:43:56 +0200 wenzelm unified Args.T with OuterLex.token;
Sat, 09 Aug 2008 22:43:55 +0200 wenzelm unified Args.T with OuterLex.token, renamed some operations;
Sat, 09 Aug 2008 22:43:54 +0200 wenzelm unified Args.T with OuterLex.token, renamed some operations;
Sat, 09 Aug 2008 22:43:53 +0200 wenzelm unified Args.T with OuterLex.token;
Sat, 09 Aug 2008 22:43:52 +0200 wenzelm load args.ML later (after outer_parse.ML);
Sat, 09 Aug 2008 22:43:46 +0200 wenzelm unified Args.T with OuterLex.token, renamed some operations;
Sat, 09 Aug 2008 12:28:13 +0200 wenzelm read_asts: report literal tokens;
Sat, 09 Aug 2008 12:28:12 +0200 wenzelm tuned error message;
Sat, 09 Aug 2008 12:28:11 +0200 wenzelm pos_of_token: Position.T;
Sat, 09 Aug 2008 12:28:10 +0200 wenzelm dest: sort strings;
Sat, 09 Aug 2008 12:28:09 +0200 wenzelm added literal;
Sat, 09 Aug 2008 00:09:39 +0200 wenzelm read_token: more robust handling of empty text;
Sat, 09 Aug 2008 00:09:38 +0200 wenzelm datatype token: maintain range, tuned representation;
Sat, 09 Aug 2008 00:09:36 +0200 wenzelm datatype token: maintain range, tuned representation;
Sat, 09 Aug 2008 00:09:35 +0200 wenzelm datatype token: maintain range, tuned representation;
Sat, 09 Aug 2008 00:09:34 +0200 wenzelm tuned SymbolPos interface;
Sat, 09 Aug 2008 00:09:31 +0200 wenzelm YXML.parse: allow text without markup, potentially empty;
Sat, 09 Aug 2008 00:09:29 +0200 wenzelm added content;
Sat, 09 Aug 2008 00:09:26 +0200 wenzelm added distance_of (permissive version);
Fri, 08 Aug 2008 19:29:01 +0200 wenzelm count offset as well;
Fri, 08 Aug 2008 19:28:59 +0200 wenzelm added offset/end_offset;
Fri, 08 Aug 2008 16:54:33 +0200 wenzelm tuned formatting;
Fri, 08 Aug 2008 15:36:40 +0200 krauss clean up dead code
Fri, 08 Aug 2008 13:36:44 +0200 wenzelm made SML/NJ happy;
Fri, 08 Aug 2008 09:44:16 +0200 krauss FundefLib.try_proof : attempt a proof and see if it works
Fri, 08 Aug 2008 09:26:15 +0200 nipkow added lemmas
Thu, 07 Aug 2008 23:56:45 +0200 wenzelm inner_syntax markup is back;
Thu, 07 Aug 2008 23:32:49 +0200 wenzelm disabled inner_syntax markup for now;
Thu, 07 Aug 2008 22:32:03 +0200 wenzelm added read_token -- with optional YXML encoding of position;
Thu, 07 Aug 2008 22:32:01 +0200 wenzelm parse_token: use Syntax.read_token, pass full position information;
Thu, 07 Aug 2008 21:13:01 +0200 wenzelm tuned;
Thu, 07 Aug 2008 21:07:57 +0200 wenzelm map_default: more explicit scope;
Thu, 07 Aug 2008 21:07:55 +0200 wenzelm datatype lexicon: alternative representation using nested Symtab.table;
Thu, 07 Aug 2008 19:21:43 +0200 wenzelm simplified Antiquote signature;
Thu, 07 Aug 2008 19:21:42 +0200 wenzelm more precise positions due to SymbolsPos.implode_delim;
Thu, 07 Aug 2008 19:21:41 +0200 wenzelm simplified Antiq: regular SymbolPos.text with position;
Thu, 07 Aug 2008 19:21:40 +0200 wenzelm renamed SymbolPos.scan_position to SymbolPos.scan_pos;
Thu, 07 Aug 2008 19:21:39 +0200 wenzelm only increment column if valid;
Thu, 07 Aug 2008 19:21:38 +0200 wenzelm install_pp Position.T;
Thu, 07 Aug 2008 19:21:37 +0200 wenzelm Position.start;
Thu, 07 Aug 2008 13:45:15 +0200 wenzelm SymbolPos.explode;
Thu, 07 Aug 2008 13:45:13 +0200 wenzelm improved position handling due to SymbolPos.T;
Thu, 07 Aug 2008 13:45:11 +0200 wenzelm improved position handling due to SymbolPos.T;
Thu, 07 Aug 2008 13:45:09 +0200 wenzelm Antiquote.read/read_arguments;
Thu, 07 Aug 2008 13:45:07 +0200 wenzelm updated type of nested sources;
Thu, 07 Aug 2008 13:45:05 +0200 wenzelm improved position handling due to SymbolPos.T;
Thu, 07 Aug 2008 13:45:03 +0200 wenzelm adapted Scan.extend_lexicon/merge_lexicons;
Thu, 07 Aug 2008 13:44:56 +0200 wenzelm renamed scan_antiquotes to read;
Thu, 07 Aug 2008 13:44:52 +0200 wenzelm export not_eof;
Thu, 07 Aug 2008 13:44:47 +0200 wenzelm reorganized lexicon: allow scanning of annotated symbols, tuned representation and interfaces;
Thu, 07 Aug 2008 13:44:42 +0200 wenzelm advance: single argument (again);
Thu, 07 Aug 2008 13:44:36 +0200 wenzelm Symbols with explicit position information.
Thu, 07 Aug 2008 13:44:33 +0200 wenzelm added General/symbol_pos.ML;
Wed, 06 Aug 2008 16:41:40 +0200 ballarin Interpretation command (theory/proof context) no longer simplifies goal.
Wed, 06 Aug 2008 13:57:25 +0200 nipkow added lemma
Wed, 06 Aug 2008 10:43:42 +0200 wenzelm made SML/NJ happy;
Wed, 06 Aug 2008 00:58:27 +0200 berghofe Reverted last change, since it caused incompatibilities.
Wed, 06 Aug 2008 00:12:31 +0200 wenzelm fall back on P.term_group, to avoid problems with inner_syntax markup (due to CodeName.read_const_exprs);
Wed, 06 Aug 2008 00:12:26 +0200 wenzelm T.end_position_of;
Wed, 06 Aug 2008 00:12:21 +0200 wenzelm adapted Antiq;
Wed, 06 Aug 2008 00:12:02 +0200 wenzelm parse_sort/typ/term/prop: report markup;
Wed, 06 Aug 2008 00:11:12 +0200 wenzelm sort/typ/term/prop: inner_syntax markup encodes original source position;
Wed, 06 Aug 2008 00:10:31 +0200 wenzelm removed obsolete range_of (already included in position);
Wed, 06 Aug 2008 00:10:22 +0200 wenzelm report markup;
Wed, 06 Aug 2008 00:10:18 +0200 wenzelm Antiq: inner vs. outer position;
Wed, 06 Aug 2008 00:10:13 +0200 wenzelm of_properties: observe Markup.position_properties';
Wed, 06 Aug 2008 00:10:08 +0200 wenzelm added position_properties';
Tue, 05 Aug 2008 19:29:09 +0200 wenzelm token: maintain of source, which retains original position information;
Tue, 05 Aug 2008 19:29:08 +0200 wenzelm moved OuterLex.count here;
Tue, 05 Aug 2008 19:29:07 +0200 wenzelm improved recover: also resync on symbol/comment/verbatim delimiters;
Tue, 05 Aug 2008 19:29:06 +0200 wenzelm advance: operate on symbol list (less overhead);
Tue, 05 Aug 2008 19:29:02 +0200 wenzelm added token;
Tue, 05 Aug 2008 14:40:48 +0200 krauss fix HOL/ex/LexOrds.thy; add to regression
Tue, 05 Aug 2008 13:31:38 +0200 wenzelm added report;
Tue, 05 Aug 2008 13:31:36 +0200 wenzelm removed axiom;
Tue, 05 Aug 2008 13:31:35 +0200 wenzelm get_fact: report position;
Tue, 05 Aug 2008 13:31:31 +0200 wenzelm Facts.lookup: return static/dynamic status;
Mon, 04 Aug 2008 22:55:10 +0200 wenzelm position scanner: encode token range;
Mon, 04 Aug 2008 22:55:08 +0200 wenzelm added encode_range;
Mon, 04 Aug 2008 22:55:04 +0200 wenzelm added end_line, end_column properties;
Mon, 04 Aug 2008 22:55:00 +0200 wenzelm meta_subst: xsymbols make it work with clean Pure;
Mon, 04 Aug 2008 21:24:19 +0200 wenzelm abstract type Scan.stopper, position taken from last input token;
Mon, 04 Aug 2008 21:24:17 +0200 wenzelm abstract type Scan.stopper;
Mon, 04 Aug 2008 21:24:15 +0200 wenzelm abstract type stopper, may depend on final input;
Mon, 04 Aug 2008 20:27:40 +0200 wenzelm removed obsolete apply_theorems(_i);
Mon, 04 Aug 2008 20:27:39 +0200 wenzelm tuned signature;
Mon, 04 Aug 2008 20:27:38 +0200 wenzelm removed obsolete note_thms_cmd;
Mon, 04 Aug 2008 20:27:37 +0200 wenzelm simplified defer_recdef(_i): plain facts via Attrib.eval_thms;
Mon, 04 Aug 2008 20:19:59 +0200 wenzelm tuned description;
Mon, 04 Aug 2008 19:25:59 +0200 wenzelm replaced mercurial.cgi by hgwebdir.cgi, resulting in http://isabelle.in.tum.de/repos/isabelle/
Mon, 04 Aug 2008 18:57:35 +0200 berghofe Quoted terms in consts_code declarations are now preprocessed as well.
Mon, 04 Aug 2008 18:56:55 +0200 berghofe Exported eval_wrapper.
Mon, 04 Aug 2008 18:56:22 +0200 berghofe - corrected bogus comment for function inst_conj_all
Mon, 04 Aug 2008 18:24:27 +0200 krauss removed dead code
Mon, 04 Aug 2008 17:13:34 +0200 wenzelm simplified prepare_command;
Mon, 04 Aug 2008 17:13:33 +0200 wenzelm Isar.command: explicitly set transaction position, as required for prepare_command errors;
Mon, 04 Aug 2008 10:37:33 +0200 ballarin Updated locale tests.
Fri, 01 Aug 2008 18:10:52 +0200 ballarin Generalised polynomial lemmas from cring to ring.
Fri, 01 Aug 2008 17:41:37 +0200 ballarin Removed import and lparams from locale record.
Fri, 01 Aug 2008 12:57:50 +0200 nipkow made setsum executable on int.
Thu, 31 Jul 2008 09:49:21 +0200 ballarin Tuned (for the sake of a meaningless log entry).
Wed, 30 Jul 2008 19:03:33 +0200 ballarin New locales for orders and lattices where the equivalence relation is not restricted to equality.
Wed, 30 Jul 2008 16:07:00 +0200 nipkow added hint about writing "x : set xs".
Wed, 30 Jul 2008 07:34:01 +0200 haftmann simple lifters
Wed, 30 Jul 2008 07:34:00 +0200 haftmann dropped imperative monad bind
Wed, 30 Jul 2008 07:33:59 +0200 haftmann facts_of
Wed, 30 Jul 2008 07:33:58 +0200 haftmann improved morphism
Wed, 30 Jul 2008 07:33:57 +0200 haftmann SML_imp, OCaml_imp
Wed, 30 Jul 2008 07:33:56 +0200 haftmann clarified
Wed, 30 Jul 2008 07:33:55 +0200 haftmann tuned
Tue, 29 Jul 2008 17:50:48 +0200 ballarin Zorn's Lemma for partial orders.
Tue, 29 Jul 2008 17:50:12 +0200 ballarin Definitions and some lemmas for reflexive orderings.
Tue, 29 Jul 2008 17:49:26 +0200 ballarin Lemmas added
Tue, 29 Jul 2008 16:19:49 +0200 ballarin New theory on divisibility.
Tue, 29 Jul 2008 16:19:19 +0200 ballarin Renamed theorems;
Tue, 29 Jul 2008 16:17:45 +0200 ballarin New theorems on summation.
Tue, 29 Jul 2008 16:17:13 +0200 ballarin Unit_inv_l, Unit_inv_r made [simp].
Tue, 29 Jul 2008 16:16:10 +0200 ballarin New theory on divisibility;
Tue, 29 Jul 2008 16:14:56 +0200 ballarin Unit_inv_l, Unit_inv_r made [simp];
Tue, 29 Jul 2008 14:20:22 +0200 haftmann Haskell now living in the RealWorld
Tue, 29 Jul 2008 14:07:23 +0200 haftmann corrected Pure dependency
Tue, 29 Jul 2008 13:16:54 +0200 nipkow added removeAll
Tue, 29 Jul 2008 08:15:44 +0200 haftmann tuned; explicit export of element accessors
Tue, 29 Jul 2008 08:15:40 +0200 haftmann PureThy: dropped note_thmss_qualified, dropped _i suffix
Tue, 29 Jul 2008 08:15:39 +0200 haftmann some steps towards explicit class target for canonical interpretation
Tue, 29 Jul 2008 08:15:38 +0200 haftmann declare
Mon, 28 Jul 2008 20:49:07 +0200 nipkow *** empty log message ***
Sun, 27 Jul 2008 20:08:16 +0200 urbanc simplified a proof
Sat, 26 Jul 2008 09:00:26 +0200 haftmann tuned function name
Sat, 26 Jul 2008 09:00:25 +0200 haftmann tuned bootstrap order
Fri, 25 Jul 2008 12:03:37 +0200 haftmann subclass now also works for subclasses with empty specificaton
Fri, 25 Jul 2008 12:03:36 +0200 haftmann dropped PureThy.note; added PureThy.add_thm
Fri, 25 Jul 2008 12:03:34 +0200 haftmann added class preorder
Fri, 25 Jul 2008 12:03:32 +0200 haftmann dropped locale (open)
Fri, 25 Jul 2008 12:03:31 +0200 haftmann added explicit root theory; some tuning
Fri, 25 Jul 2008 12:03:28 +0200 haftmann tuned
Fri, 25 Jul 2008 07:35:53 +0200 haftmann dropped locale (open)
Mon, 21 Jul 2008 16:30:49 +0200 haftmann (re-)added simp rules for (_ + _) div/mod _
Mon, 21 Jul 2008 15:27:23 +0200 haftmann (re-)added simp rules for (_ + _) div/mod _
Mon, 21 Jul 2008 15:26:26 +0200 haftmann added explicit purge_data
Mon, 21 Jul 2008 15:26:25 +0200 haftmann added code generation
Mon, 21 Jul 2008 15:26:24 +0200 haftmann fixed code generator setup
Mon, 21 Jul 2008 15:26:23 +0200 haftmann (adjusted)
Mon, 21 Jul 2008 13:37:14 +0200 chaieb Tuned and corrected ideal_tac for algebra.
Mon, 21 Jul 2008 13:37:10 +0200 chaieb Theorems divides_le, ind_euclid, bezout_lemma, bezout_add, bezout, bezout_add_strong, gcd_unique,gcd_eq, bezout_gcd, bezout_gcd_strong, gcd_mult_distrib, gcd_bezout to GCD.thy
Mon, 21 Jul 2008 13:37:05 +0200 chaieb Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
Mon, 21 Jul 2008 13:36:59 +0200 chaieb Tuned and simplified proofs
Mon, 21 Jul 2008 13:36:44 +0200 chaieb Added theorems zmod_eq_dvd_iff and nat_mod_eq_iff previously in Pocklington.thy --- relevant for algebra
Mon, 21 Jul 2008 13:36:39 +0200 chaieb Relevant rules added to algebra's context
Sun, 20 Jul 2008 23:07:03 +0200 wenzelm renamed item to span, renamed contructors;
Sun, 20 Jul 2008 23:07:01 +0200 wenzelm adapted ThyEdit.span;
Sun, 20 Jul 2008 23:06:59 +0200 wenzelm maintain token range;
Sun, 20 Jul 2008 23:06:58 +0200 wenzelm tty loop: do not report status;
Sun, 20 Jul 2008 23:06:55 +0200 wenzelm added type range;
Sun, 20 Jul 2008 23:06:53 +0200 wenzelm renamed command span markup;
Sun, 20 Jul 2008 20:23:49 +0200 wenzelm SideKickParsedData: minimal content;
Sun, 20 Jul 2008 11:19:08 +0200 haftmann (adjusted)
Sun, 20 Jul 2008 11:10:04 +0200 haftmann (adjusted)
Sat, 19 Jul 2008 19:27:13 +0200 bulwahn added verification framework for the HeapMonad and quicksort as example for this framework
Sat, 19 Jul 2008 11:05:18 +0200 wenzelm build jedit plugin only if jedit is available;
Fri, 18 Jul 2008 22:03:20 +0200 wenzelm misc tuning;
Fri, 18 Jul 2008 18:25:57 +0200 haftmann more class instantiations
Fri, 18 Jul 2008 18:25:56 +0200 haftmann refined code generator setup for rational numbers; more simplification rules for rational numbers
Fri, 18 Jul 2008 18:25:53 +0200 haftmann moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
Fri, 18 Jul 2008 17:09:48 +0200 wenzelm fixed Scala path;
Thu, 17 Jul 2008 21:24:26 +0200 wenzelm tuned build order;
Thu, 17 Jul 2008 21:23:32 +0200 wenzelm proper purge_tmp;
Thu, 17 Jul 2008 21:23:08 +0200 wenzelm tuned message;
Thu, 17 Jul 2008 21:22:44 +0200 wenzelm tuned line breaks (NB: generated text is inserted here);
Thu, 17 Jul 2008 21:07:17 +0200 wenzelm proper usage message;
Thu, 17 Jul 2008 20:40:05 +0200 wenzelm make Isabelle source distribution (via Mercurial);
Thu, 17 Jul 2008 20:15:15 +0200 wenzelm explicit Distribution.changelog;
Thu, 17 Jul 2008 20:15:14 +0200 wenzelm structure Distribution: swapped default for is_official;
Thu, 17 Jul 2008 20:15:13 +0200 wenzelm ThyInfo.remove_thy;
Thu, 17 Jul 2008 20:15:12 +0200 wenzelm structure Distribution: swapped default for is_official;
Thu, 17 Jul 2008 20:05:19 +0200 wenzelm use ../isabelle.sty and ../isabellesym.sty;
Thu, 17 Jul 2008 17:11:34 +0200 wenzelm tuned whitespace;
Thu, 17 Jul 2008 17:10:53 +0200 wenzelm removed old checklist;
Thu, 17 Jul 2008 17:03:48 +0200 wenzelm obsolete;
Thu, 17 Jul 2008 17:01:54 +0200 wenzelm tuned;
Thu, 17 Jul 2008 16:56:50 +0200 wenzelm discontinued maketags;
Thu, 17 Jul 2008 16:56:48 +0200 wenzelm assume GNU tar and find;
Thu, 17 Jul 2008 16:19:06 +0200 wenzelm tuned;
Thu, 17 Jul 2008 16:17:05 +0200 wenzelm use ../isabellesym.sty, which is always available;
Thu, 17 Jul 2008 15:35:15 +0200 wenzelm Admin/build browser;
(0) -10000 -3000 -1000 -256 +256 +1000 +3000 +10000 +30000 tip