Wed, 21 Sep 2005 12:03:41 +0200 berghofe Added new "value" command.
Wed, 21 Sep 2005 12:02:56 +0200 berghofe Simplified code generator for numerals.
Wed, 21 Sep 2005 12:02:19 +0200 berghofe Declared nat_number_of as code lemma.
Wed, 21 Sep 2005 12:01:31 +0200 berghofe - Added eval_term function and value command
Wed, 21 Sep 2005 11:50:52 +0200 wenzelm tunes;
Wed, 21 Sep 2005 11:50:38 +0200 wenzelm updated for Isabelle2005;
Wed, 21 Sep 2005 11:50:20 +0200 wenzelm HOL-Complex-Matrix: fixed deps;
Wed, 21 Sep 2005 11:49:31 +0200 wenzelm tuned;
Wed, 21 Sep 2005 11:19:16 +0200 wenzelm updated for Isabelle2005;
Wed, 21 Sep 2005 10:40:28 +0200 wenzelm tuned;
Wed, 21 Sep 2005 10:39:38 +0200 haftmann (name mess cleanup)
Wed, 21 Sep 2005 10:33:59 +0200 haftmann introduced AList module
Wed, 21 Sep 2005 10:32:24 +0200 haftmann removed assoc, overwrite
Wed, 21 Sep 2005 10:32:06 +0200 haftmann added update_warn
Wed, 21 Sep 2005 00:07:32 +0200 wenzelm tuned;
Tue, 20 Sep 2005 23:36:57 +0200 wenzelm fixed proof script of lemma merges_same_conv (Why did it stop working?);
Tue, 20 Sep 2005 22:07:36 +0200 wenzelm updated;
Tue, 20 Sep 2005 22:02:06 +0200 wenzelm tuned;
Tue, 20 Sep 2005 21:51:06 +0200 wenzelm HOL/ex/Chinese.thy;
Tue, 20 Sep 2005 21:48:47 +0200 wenzelm tuned;
Tue, 20 Sep 2005 21:48:37 +0200 wenzelm more contributions;
Tue, 20 Sep 2005 21:39:00 +0200 wenzelm tuned headers;
Tue, 20 Sep 2005 21:34:20 +0200 wenzelm tuned header;
Tue, 20 Sep 2005 21:09:41 +0200 wenzelm use "ML-Systems/smlnj-basis-compat.ML" *after* Interrupt;
Tue, 20 Sep 2005 20:16:55 +0200 wenzelm fixed proof script of lemma Cond_sound (Why did it stop working anyway?);
Tue, 20 Sep 2005 19:38:35 +0200 webertj bugfix in "zchaff_with_proofs"
Tue, 20 Sep 2005 18:47:42 +0200 paulson fixed recursive-looking declaration
Tue, 20 Sep 2005 18:43:39 +0200 paulson tidying, and support for axclass/classrel clauses
Tue, 20 Sep 2005 18:42:56 +0200 paulson fixed syntax for sml/nj
Tue, 20 Sep 2005 17:01:43 +0200 webertj undone the previous change: show_hyps not supported anymore
Tue, 20 Sep 2005 16:19:51 +0200 webertj pointers to src/HOL/Tools/sat_solver.ML added in comments
Tue, 20 Sep 2005 16:17:34 +0200 haftmann introduced AList module in favor of assoc etc.
Tue, 20 Sep 2005 15:12:40 +0200 webertj new menu item show-sort-hypotheses to toggle show_hyps
Tue, 20 Sep 2005 14:20:58 +0200 wenzelm HOL/ex/Chinese.thy;
Tue, 20 Sep 2005 14:17:31 +0200 wenzelm HOL-ex: Library/Commutative_Ring.thy;
Tue, 20 Sep 2005 14:13:20 +0200 wenzelm moved Tools/comm_ring.ML to Library;
Tue, 20 Sep 2005 14:10:29 +0200 wenzelm added Commutative_Ring (from Main HOL);
Tue, 20 Sep 2005 14:06:00 +0200 wenzelm Simplifier.inherit_bounds;
Tue, 20 Sep 2005 14:04:34 +0200 wenzelm TextIO.inputLine: handle IO.Io, assuming it stems from a signal;
Tue, 20 Sep 2005 14:03:42 +0200 wenzelm get_interrupt: special handling of IO.io now in ML-Systems/smlnj-basis-compat.ML;
Tue, 20 Sep 2005 14:03:41 +0200 wenzelm removed obsolete thms_containing;
Tue, 20 Sep 2005 14:03:40 +0200 wenzelm tuned;
Tue, 20 Sep 2005 14:03:39 +0200 wenzelm tuned simprocs;
Tue, 20 Sep 2005 14:03:38 +0200 wenzelm removed Commutative_Ring hacks;
Tue, 20 Sep 2005 14:03:37 +0200 wenzelm tuned theory dependencies;
Tue, 20 Sep 2005 13:58:58 +0200 wenzelm removed Commutative_Ring.thy, added HOL/ex/Chinese.thy;
Tue, 20 Sep 2005 13:57:08 +0200 wenzelm tuned;
Tue, 20 Sep 2005 13:56:34 +0200 wenzelm Chinese Unicode example;
Tue, 20 Sep 2005 13:56:01 +0200 wenzelm tuned proofs;
Tue, 20 Sep 2005 13:33:27 +0200 chaieb The simpset of the actual theory is take, in order to handle rings defined after the method
Tue, 20 Sep 2005 13:17:55 +0200 paulson further tidying; killing of old Watcher loops
Tue, 20 Sep 2005 13:17:55 +0200 nipkow added a number of lemmas
Tue, 20 Sep 2005 13:17:32 +0200 paulson uniform handling of interrupts
Tue, 20 Sep 2005 10:36:33 +0200 chaieb algebra method added.
Tue, 20 Sep 2005 08:24:18 +0200 haftmann improved eq_fst and eq_snd, removed some deprecated stuff
Tue, 20 Sep 2005 08:23:59 +0200 haftmann added make and find
Tue, 20 Sep 2005 08:21:49 +0200 haftmann slight adaptions to library changes
Tue, 20 Sep 2005 08:20:22 +0200 haftmann infix operator precedence
Tue, 20 Sep 2005 00:16:29 +0200 webertj using curried Inttab.update_new function now
Mon, 19 Sep 2005 23:45:59 +0200 webertj SAT solver interface modified to support proofs of unsatisfiability
Mon, 19 Sep 2005 23:23:51 +0200 wenzelm shrink: compress terms and types;
Mon, 19 Sep 2005 23:22:51 +0200 wenzelm added String.isSuffix;
Mon, 19 Sep 2005 22:35:39 +0200 obua maybe the last bug fix (sigh)?
Mon, 19 Sep 2005 19:49:09 +0200 obua Removed superfluous HOL/Matrix/cplex/ROOT.ML.
Mon, 19 Sep 2005 18:30:22 +0200 paulson further simplification of the Isabelle-ATP linkup
Mon, 19 Sep 2005 16:42:11 +0200 haftmann added make function
Mon, 19 Sep 2005 16:39:27 +0200 haftmann removed some deprecated assocation list functions
Mon, 19 Sep 2005 16:38:35 +0200 haftmann introduced AList module
Mon, 19 Sep 2005 15:12:13 +0200 paulson simplification of the Isabelle-ATP code; hooks for batch generation of problems
Mon, 19 Sep 2005 14:20:45 +0200 kleing update usage message
Mon, 19 Sep 2005 12:05:08 +0200 wenzelm obsolete;
Sun, 18 Sep 2005 15:20:08 +0200 wenzelm converted to Isar theory format;
Sun, 18 Sep 2005 14:25:48 +0200 wenzelm converted to Isar theory format;
Sat, 17 Sep 2005 20:49:14 +0200 wenzelm converted to Isar theory format;
Sat, 17 Sep 2005 20:16:35 +0200 wenzelm tuned;
Sat, 17 Sep 2005 20:14:30 +0200 wenzelm converted to Isar theory format;
Sat, 17 Sep 2005 19:17:35 +0200 wenzelm moved quick_and_dirty to Pure/ROOT.ML;
Sat, 17 Sep 2005 19:17:34 +0200 wenzelm pretty_thm_aux: ora masked by quick_and_dirty;
Sat, 17 Sep 2005 19:17:33 +0200 wenzelm added quick_and_dirty (from Isar/skip_proofs.ML);
Sat, 17 Sep 2005 19:12:58 +0200 wenzelm manually generated from Isabelle/HOLCF/IOA/Complex/Import;
Sat, 17 Sep 2005 18:25:11 +0200 wenzelm tuned document;
Sat, 17 Sep 2005 18:24:57 +0200 wenzelm tuned;
Sat, 17 Sep 2005 18:11:30 +0200 wenzelm added with_charset: string -> ('a -> 'b) -> 'a -> 'b;
Sat, 17 Sep 2005 18:11:29 +0200 wenzelm tuned comments;
Sat, 17 Sep 2005 18:11:28 +0200 wenzelm pretty_thm_aux: aconv hyps;
Sat, 17 Sep 2005 18:11:27 +0200 wenzelm removed obsolete BasisLibrary;
Sat, 17 Sep 2005 18:11:26 +0200 wenzelm Hebrew: HTML.with_charset;
Sat, 17 Sep 2005 18:11:25 +0200 wenzelm removed obsolete BasisLibrary;
Sat, 17 Sep 2005 18:11:24 +0200 wenzelm added quickcheck_params (from Main.thy);
Sat, 17 Sep 2005 18:11:23 +0200 wenzelm removed spurious PolyML.exception_trace;
Sat, 17 Sep 2005 18:11:22 +0200 wenzelm moved setup ResAxioms.clause_setup to Main.thy (it refers to all previous theories);
Sat, 17 Sep 2005 18:11:21 +0200 wenzelm minor cleanup, moved stuff in its proper place;
Sat, 17 Sep 2005 18:11:20 +0200 wenzelm generate: added HOL-Complex-Generate-HOLLight;
Sat, 17 Sep 2005 18:11:19 +0200 wenzelm added code generator setup (from Main.thy);
Sat, 17 Sep 2005 18:11:18 +0200 wenzelm lemmas [code] = imp_conv_disj (from Main.thy) -- Why does it need Datatype?
Sat, 17 Sep 2005 18:11:17 +0200 wenzelm HTML.with_charset;
Sat, 17 Sep 2005 17:35:26 +0200 wenzelm converted to Isar theory format;
Sat, 17 Sep 2005 14:02:31 +0200 wenzelm tuned document;
Sat, 17 Sep 2005 12:51:03 +0200 wenzelm obsolete;
Sat, 17 Sep 2005 12:50:57 +0200 wenzelm plain test session, includes example;
Sat, 17 Sep 2005 12:18:08 +0200 wenzelm theory_to_proof: check theory of initial proof state, which must not be changed;
Sat, 17 Sep 2005 12:18:07 +0200 wenzelm added auto_fix (from proof.ML);
Sat, 17 Sep 2005 12:18:06 +0200 wenzelm export put_facts;
Sat, 17 Sep 2005 12:18:05 +0200 wenzelm interpretation: use goal commands without target -- no storing of results;
Sat, 17 Sep 2005 12:18:04 +0200 wenzelm theorem(_i): empty target;
Sat, 17 Sep 2005 12:18:03 +0200 wenzelm pretty_thm_aux: observe asms context;
Sat, 17 Sep 2005 12:18:02 +0200 wenzelm tuned;
Sat, 17 Sep 2005 12:18:00 +0200 wenzelm Cube: converted to Isar, use locales;
Sat, 17 Sep 2005 11:49:29 +0200 obua 1) mapped .. and == constants
Sat, 17 Sep 2005 01:50:01 +0200 huffman use interpretation command
Fri, 16 Sep 2005 23:55:23 +0200 huffman add HOLCF entries for pcpodef, cont_proc, fixrec;
Fri, 16 Sep 2005 23:01:29 +0200 wenzelm converted to Isar theory format;
Fri, 16 Sep 2005 21:02:15 +0200 obua fixed HOL-light/Isabelle syntax incompatability via more protect_xxx functions
Fri, 16 Sep 2005 20:30:44 +0200 huffman add header
Fri, 16 Sep 2005 16:07:22 +0200 ballarin tuned
Fri, 16 Sep 2005 14:46:31 +0200 ballarin interpretation uses primitive goal interface
Fri, 16 Sep 2005 14:44:52 +0200 ballarin tuned
Fri, 16 Sep 2005 11:39:09 +0200 paulson PARTIAL conversion to Vampire8
Fri, 16 Sep 2005 11:38:49 +0200 paulson catching exception Io
Fri, 16 Sep 2005 02:20:50 +0200 huffman rearranged
(0) -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip