wenzelm [Tue, 23 Oct 2001 22:59:14 +0200] rev 11915
print fixed names as plain strings;
wenzelm [Tue, 23 Oct 2001 22:58:15 +0200] rev 11914
eliminated old numerals;
wenzelm [Tue, 23 Oct 2001 22:57:52 +0200] rev 11913
use generic 1 instead of Numeral1;
use improved iff declaration;
tuned;
wenzelm [Tue, 23 Oct 2001 22:56:55 +0200] rev 11912
eliminated Numeral0;
wenzelm [Tue, 23 Oct 2001 22:54:01 +0200] rev 11911
build option enables most basic browser info (for proper recording of session);
wenzelm [Tue, 23 Oct 2001 22:53:08 +0200] rev 11910
build option;
wenzelm [Tue, 23 Oct 2001 22:52:45 +0200] rev 11909
tuned;
wenzelm [Tue, 23 Oct 2001 22:52:31 +0200] rev 11908
eliminated old numerals;
wenzelm [Tue, 23 Oct 2001 22:51:30 +0200] rev 11907
pass build mode to process;
wenzelm [Tue, 23 Oct 2001 19:15:00 +0200] rev 11906
removed export_thm;
wenzelm [Tue, 23 Oct 2001 19:14:47 +0200] rev 11905
trace_rules: only non-empty;
wenzelm [Tue, 23 Oct 2001 19:14:31 +0200] rev 11904
removed obsolete "exported" att;
wenzelm [Tue, 23 Oct 2001 19:14:13 +0200] rev 11903
replace_dummy_patterns: lift over bounds;
wenzelm [Tue, 23 Oct 2001 19:13:44 +0200] rev 11902
iff: always rotate prems;
wenzelm [Tue, 23 Oct 2001 19:13:17 +0200] rev 11901
apply(simp add: three_def numerals) (* FIXME !? *);
wenzelm [Tue, 23 Oct 2001 19:12:58 +0200] rev 11900
unset DISPLAY (again);
wenzelm [Tue, 23 Oct 2001 19:12:37 +0200] rev 11899
* Pure: removed obsolete 'exported' attribute;
* Pure: dummy pattern "_" in is/let is now automatically ``lifted''
over bound variables: "ALL x. P x --> Q x" (is "ALL x. _ --> ?C x")
supersedes more cumbersome ... (is "ALL x. _ x --> ?C x");
wenzelm [Mon, 22 Oct 2001 23:39:00 +0200] rev 11898
*** empty log message ***
wenzelm [Mon, 22 Oct 2001 18:07:53 +0200] rev 11897
moved object_logic.ML to Isar/object_logic.ML;
wenzelm [Mon, 22 Oct 2001 18:07:30 +0200] rev 11896
moved locale.ML to Isar/locale.ML;
wenzelm [Mon, 22 Oct 2001 18:04:26 +0200] rev 11895
moved goal related stuff to goals.ML;
wenzelm [Mon, 22 Oct 2001 18:04:11 +0200] rev 11894
Display.current_goals_markers;
wenzelm [Mon, 22 Oct 2001 18:04:00 +0200] rev 11893
tuned;
wenzelm [Mon, 22 Oct 2001 18:03:49 +0200] rev 11892
moved prove_goalw_cterm to goals.ML;
cleaned up;
wenzelm [Mon, 22 Oct 2001 18:03:21 +0200] rev 11891
moved local defs to proof.ML (for locales);
wenzelm [Mon, 22 Oct 2001 18:02:50 +0200] rev 11890
improved source arrangement of obtain;
wenzelm [Mon, 22 Oct 2001 18:02:21 +0200] rev 11889
rearrange sources for locales;
wenzelm [Mon, 22 Oct 2001 18:02:04 +0200] rev 11888
Display.print_current_goals_fn;
wenzelm [Mon, 22 Oct 2001 18:01:52 +0200] rev 11887
Display.print_goals;
wenzelm [Mon, 22 Oct 2001 18:01:38 +0200] rev 11886
Display.pretty_thms;
wenzelm [Mon, 22 Oct 2001 18:01:26 +0200] rev 11885
qualified names;
wenzelm [Mon, 22 Oct 2001 18:01:15 +0200] rev 11884
make this module appeat late in Pure;
moved print_current_goals to display.ML;
added quick_and_dirty_prove_goalw_cterm (from Isar/skip_proof.ML);
added thm database functions (from Thy/thm_database.ML);
wenzelm [Mon, 22 Oct 2001 17:59:39 +0200] rev 11883
print_goals stuff is back (from locale.ML);
wenzelm [Mon, 22 Oct 2001 17:58:56 +0200] rev 11882
reorganize sources to accomodate locales;
wenzelm [Mon, 22 Oct 2001 17:58:37 +0200] rev 11881
corollary;
wenzelm [Mon, 22 Oct 2001 17:58:26 +0200] rev 11880
quick_and_dirty_prove_goalw_cterm;
wenzelm [Mon, 22 Oct 2001 17:58:11 +0200] rev 11879
javac -depend;
wenzelm [Mon, 22 Oct 2001 17:56:16 +0200] rev 11878
-D generated;
berghofe [Mon, 22 Oct 2001 14:58:05 +0200] rev 11877
Added "clean" target.
berghofe [Mon, 22 Oct 2001 14:55:16 +0200] rev 11876
Fixed problem with batch mode layout, which caused an AWT exception when
no X11 connection was available.
berghofe [Mon, 22 Oct 2001 14:53:52 +0200] rev 11875
initBrowser now has additional noAWT argument.
berghofe [Mon, 22 Oct 2001 14:52:43 +0200] rev 11874
Constructor no longer takes font as an argument.
berghofe [Mon, 22 Oct 2001 14:52:12 +0200] rev 11873
Moved font settings from TreeNode to TreeBrowser.
berghofe [Mon, 22 Oct 2001 14:51:39 +0200] rev 11872
Moved font settings from Vertex to GraphView.
paulson [Mon, 22 Oct 2001 12:11:00 +0200] rev 11871
deleted the redundant first argument of adjust(a,b)
paulson [Mon, 22 Oct 2001 12:01:35 +0200] rev 11870
Numerals now work for the integers: the binary numerals for 0 and 1 rewrite
to their abstract counterparts, while other binary numerals work correctly.
paulson [Mon, 22 Oct 2001 11:55:35 +0200] rev 11869
New simproc, needed to cope with combinations of (abstract) 0, (abstract) 1,
binary numerals in literal arithmetic.
paulson [Mon, 22 Oct 2001 11:54:22 +0200] rev 11868
Numerals now work for the integers: the binary numerals for 0 and 1 rewrite
to their abstract counterparts, while other binary numerals work correctly.
wenzelm [Mon, 22 Oct 2001 11:01:30 +0200] rev 11867
keep DISPLAY;
wenzelm [Sun, 21 Oct 2001 19:49:29 +0200] rev 11866
updated;
wenzelm [Sun, 21 Oct 2001 19:48:19 +0200] rev 11865
renamed to Typedefs.thy to avoid conflict with main HOL version;
wenzelm [Sun, 21 Oct 2001 19:44:25 +0200] rev 11864
* proper spacing of consecutive markup elements, especially text
blocks after section headings;
wenzelm [Sun, 21 Oct 2001 19:42:53 +0200] rev 11863
\newif\ifisamarkup controls spacing of isabeginpar;
wenzelm [Sun, 21 Oct 2001 19:42:24 +0200] rev 11862
improved spacing;
wenzelm [Sun, 21 Oct 2001 19:41:43 +0200] rev 11861
maintain Latex.flag_markup;
wenzelm [Sun, 21 Oct 2001 19:40:39 +0200] rev 11860
flag_markup;
wenzelm [Sun, 21 Oct 2001 19:36:12 +0200] rev 11859
Types/document/Typedefs;
wenzelm [Sun, 21 Oct 2001 19:35:40 +0200] rev 11858
renamed Typedef.thy to Typedefs.thy (former already present in main HOL);
wenzelm [Sat, 20 Oct 2001 22:07:44 +0200] rev 11857
got rid of separate root.tex;
wenzelm [Sat, 20 Oct 2001 20:23:37 +0200] rev 11856
graceful interpretation of -i/-d/-D options;
verbose: additional messages/warnings;
include document graph;
wenzelm [Sat, 20 Oct 2001 20:22:17 +0200] rev 11855
include document graph;
wenzelm [Sat, 20 Oct 2001 20:21:40 +0200] rev 11854
document graph option;
wenzelm [Sat, 20 Oct 2001 20:21:14 +0200] rev 11853
conditional: bool -> (unit -> unit) -> unit;
std_error: string -> unit;
wenzelm [Sat, 20 Oct 2001 20:20:41 +0200] rev 11852
added TextIO.stdErr;
wenzelm [Sat, 20 Oct 2001 20:20:21 +0200] rev 11851
include document graph;
tuned;
wenzelm [Sat, 20 Oct 2001 20:19:47 +0200] rev 11850
document graphs for several sessions;
wenzelm [Sat, 20 Oct 2001 20:18:57 +0200] rev 11849
tuned;
wenzelm [Sat, 20 Oct 2001 20:18:45 +0200] rev 11848
calculational rules moved from FOL to IFOL;
wenzelm [Sat, 20 Oct 2001 20:18:19 +0200] rev 11847
option -g for document graph;
removed all presumptions about -d/-D (handled by isabelle process);
wenzelm [Sat, 20 Oct 2001 20:16:55 +0200] rev 11846
option -q also excludes -v true in generated stuff;
tuned message;
wenzelm [Sat, 20 Oct 2001 20:15:44 +0200] rev 11845
dvips -q;
wenzelm [Sat, 20 Oct 2001 20:15:27 +0200] rev 11844
removed -v option (handled by isabelle process);
wenzelm [Sat, 20 Oct 2001 20:14:56 +0200] rev 11843
-o pdf: produce *both* eps and pdf;
tuned;
wenzelm [Sat, 20 Oct 2001 20:14:16 +0200] rev 11842
* greatly simplified document preparation setup, including more
graceful interpretation of isatool usedir -i/-d/-D options, and more
instructive isatool mkdir; users should basically be able to get
started with "isatool mkdir Test && isatool make";
* theory dependency graph may now be incorporated into documents;
isatool usedir -g true will produce session_graph.eps/.pdf for use
with \includegraphics of LaTeX;
wenzelm [Fri, 19 Oct 2001 22:03:25 +0200] rev 11841
got rid of ML proof scripts;
wenzelm [Fri, 19 Oct 2001 22:02:25 +0200] rev 11840
induct_method.ML -- proof by cases and induction on sets and types (Isar);
wenzelm [Fri, 19 Oct 2001 22:02:02 +0200] rev 11839
latex output: bold lambda;
wenzelm [Fri, 19 Oct 2001 22:01:25 +0200] rev 11838
got rid of ML proof scripts for Product_Type;
wenzelm [Fri, 19 Oct 2001 22:00:08 +0200] rev 11837
got rid of Provers/split_paired_all.ML;
wenzelm [Fri, 19 Oct 2001 21:59:33 +0200] rev 11836
improved default dependencies;
wenzelm [Fri, 19 Oct 2001 12:17:04 +0200] rev 11835
revert to proper version (!);
wenzelm [Thu, 18 Oct 2001 21:27:47 +0200] rev 11834
GPLed;
wenzelm [Thu, 18 Oct 2001 21:22:40 +0200] rev 11833
tuned;
wenzelm [Thu, 18 Oct 2001 21:07:29 +0200] rev 11832
use abstract product type instead of datatype;
wenzelm [Thu, 18 Oct 2001 21:05:35 +0200] rev 11831
moved atomize stuff to theory HOL;
wenzelm [Thu, 18 Oct 2001 21:03:43 +0200] rev 11830
legacy interfaces for axclass instantiation;
wenzelm [Thu, 18 Oct 2001 21:02:46 +0200] rev 11829
added map_base;
wenzelm [Thu, 18 Oct 2001 21:02:26 +0200] rev 11828
sane internal interfaces for instance;
wenzelm [Thu, 18 Oct 2001 21:01:59 +0200] rev 11827
sane internal interface for add_typedef(_i);
wenzelm [Thu, 18 Oct 2001 21:01:18 +0200] rev 11826
proper setup for abstract product types;
wenzelm [Thu, 18 Oct 2001 20:59:59 +0200] rev 11825
moved InductMethod.setup to theory HOL;
wenzelm [Thu, 18 Oct 2001 20:59:33 +0200] rev 11824
setup generic cases and induction (from Inductive.thy);
wenzelm [Wed, 17 Oct 2001 20:25:51 +0200] rev 11823
guillemot syntax;
wenzelm [Wed, 17 Oct 2001 20:25:19 +0200] rev 11822
improved internal interface of typedef;
wenzelm [Wed, 17 Oct 2001 20:24:37 +0200] rev 11821
abstract product types;
wenzelm [Wed, 17 Oct 2001 20:24:03 +0200] rev 11820
proper proof of split_paired_all (presently unused);
wenzelm [Wed, 17 Oct 2001 18:52:30 +0200] rev 11819
tuned comments;
wenzelm [Wed, 17 Oct 2001 18:51:03 +0200] rev 11818
added mk_UNIV;
wenzelm [Wed, 17 Oct 2001 18:50:49 +0200] rev 11817
tuned;
wenzelm [Tue, 16 Oct 2001 23:02:14 +0200] rev 11816
simplified exporter interface;
wenzelm [Tue, 16 Oct 2001 23:00:21 +0200] rev 11815
added implies_intr_goals;
wenzelm [Tue, 16 Oct 2001 22:59:30 +0200] rev 11814
tuned;
berghofe [Tue, 16 Oct 2001 19:56:31 +0200] rev 11813
Tuned.
berghofe [Tue, 16 Oct 2001 19:54:53 +0200] rev 11812
Removed exit command from end of main method.
berghofe [Tue, 16 Oct 2001 19:54:24 +0200] rev 11811
PS method now calculates layout using default font metrics.
berghofe [Tue, 16 Oct 2001 19:53:12 +0200] rev 11810
Inserted table for character widths.
wenzelm [Tue, 16 Oct 2001 17:58:13 +0200] rev 11809
tuned induction proofs;
wenzelm [Tue, 16 Oct 2001 17:56:12 +0200] rev 11808
dest_env: norm_term on rhs;
wenzelm [Tue, 16 Oct 2001 17:55:53 +0200] rev 11807
typedef: export result;
wenzelm [Tue, 16 Oct 2001 17:55:38 +0200] rev 11806
ignore typedef result;
wenzelm [Tue, 16 Oct 2001 17:55:16 +0200] rev 11805
declare projected induction rules stemming from nested recursion;
wenzelm [Tue, 16 Oct 2001 17:52:07 +0200] rev 11804
TypedefPackage.add_typedef_no_result;