wenzelm [Wed, 10 Oct 2012 15:17:40 +0200] rev 49753
eliminated spurious fact duplicates;
wenzelm [Wed, 10 Oct 2012 15:01:20 +0200] rev 49752
modernized dynamic "rules" -- avoid rebinding of static facts;
wenzelm [Tue, 09 Oct 2012 22:24:24 +0200] rev 49751
removed redundant lemma, cf. class zero_neq_one in HOL/Rings.thy;
wenzelm [Tue, 09 Oct 2012 21:33:12 +0200] rev 49750
clarified Element.init vs. Element.activate: refrain from hard-wiring Thm.def_binding_optional to avoid duplicate facts;
wenzelm [Tue, 09 Oct 2012 20:23:58 +0200] rev 49749
tuned;
wenzelm [Tue, 09 Oct 2012 20:05:17 +0200] rev 49748
clarified Local_Defs.add_def(s): refrain from hard-wiring Thm.def_binding_optional;
clarified Generic_Target.define: avoid duplicate def binding via Local_Defs.add_def;
wenzelm [Tue, 09 Oct 2012 19:24:19 +0200] rev 49747
more explicit flags for facts table;
wenzelm [Tue, 09 Oct 2012 15:31:45 +0200] rev 49746
minor tuning;
wenzelm [Tue, 09 Oct 2012 13:57:51 +0200] rev 49745
more conventional Double constants;
wenzelm [Tue, 09 Oct 2012 13:50:24 +0200] rev 49744
tuned source structure;
wenzelm [Tue, 09 Oct 2012 13:29:43 +0200] rev 49743
tuned;
wenzelm [Tue, 09 Oct 2012 13:27:52 +0200] rev 49742
tuned;
wenzelm [Tue, 09 Oct 2012 11:51:06 +0200] rev 49741
merged
blanchet [Tue, 09 Oct 2012 00:40:33 +0200] rev 49740
added type annotations to generated Isar proofs -- code by Steffen Smolka
haftmann [Mon, 08 Oct 2012 12:03:49 +0200] rev 49739
consolidated names of theorems on composition;
generalized former theorem UN_o;
comp_assoc orients to the right, as is more common
haftmann [Mon, 08 Oct 2012 11:37:03 +0200] rev 49738
corrected NEWS
wenzelm [Mon, 08 Oct 2012 23:29:07 +0200] rev 49737
avoid somewhat heavy rebuilding of SortedMap via map where plain iteration is sufficient;
more elementary level_list: avoid stack overflow;
prefer elementary graph operations;
tuned;
wenzelm [Mon, 08 Oct 2012 21:17:20 +0200] rev 49736
clarified long_names -- conform to usual Isabelle practice of not analysing internal names;
wenzelm [Mon, 08 Oct 2012 20:39:57 +0200] rev 49735
more precise repaint and revalidate -- the latter is important to keep in sync with content update;
wenzelm [Mon, 08 Oct 2012 14:49:04 +0200] rev 49734
tuned;
wenzelm [Mon, 08 Oct 2012 14:10:38 +0200] rev 49733
prefer synchronous Mutator_Event.Bus on Swing_Thread;
wenzelm [Mon, 08 Oct 2012 13:20:55 +0200] rev 49732
more direct tooltip content;
wenzelm [Mon, 08 Oct 2012 12:54:00 +0200] rev 49731
tuned;
wenzelm [Mon, 08 Oct 2012 12:40:35 +0200] rev 49730
use Pretty_Tooltip for Graphview_Panel;
tuned signature;
wenzelm [Mon, 08 Oct 2012 12:02:32 +0200] rev 49729
more basic tooltips;
wenzelm [Sun, 07 Oct 2012 16:26:31 +0200] rev 49728
close tooltips more thoroughly;
wenzelm [Sun, 07 Oct 2012 16:15:31 +0200] rev 49727
make buttons closer to original mouse position;
wenzelm [Sun, 07 Oct 2012 16:05:31 +0200] rev 49726
detach tooltip as dockable window;
wenzelm [Sun, 07 Oct 2012 15:05:11 +0200] rev 49725
explicit close button;
haftmann [Sat, 06 Oct 2012 16:03:41 +0200] rev 49724
congruence rule for Finite_Set.fold
haftmann [Sat, 06 Oct 2012 11:08:52 +0200] rev 49723
alternative simplification of ^^ to the righthand side;
lifting of comp_fun_commute to ^^
wenzelm [Fri, 05 Oct 2012 18:01:48 +0200] rev 49722
eliminated obsolete tooltip delay -- bypassed by Pretty_Tooltip;
wenzelm [Fri, 05 Oct 2012 14:51:33 +0200] rev 49721
merged
blanchet [Fri, 05 Oct 2012 10:57:03 +0200] rev 49720
newer versions of Z3 call it "Bool" not "bool"
haftmann [Thu, 04 Oct 2012 23:19:02 +0200] rev 49719
simplified type of msetprod;
n.b. image function need not be part of minimal definition of msetprod, since multisets may already contain repeated elements
haftmann [Thu, 04 Oct 2012 23:19:02 +0200] rev 49718
tuned proof
haftmann [Thu, 04 Oct 2012 23:19:02 +0200] rev 49717
default simp rule for image under identity
haftmann [Thu, 04 Oct 2012 23:19:02 +0200] rev 49716
dropped duplicate facts; tuned syntax
haftmann [Thu, 04 Oct 2012 23:19:02 +0200] rev 49715
more facts on setsum and setprod
traytel [Thu, 04 Oct 2012 17:26:04 +0200] rev 49714
made SML/NJ happier
traytel [Thu, 04 Oct 2012 17:16:55 +0200] rev 49713
do not expose details of internal data structures for composition of BNFs
wenzelm [Fri, 05 Oct 2012 14:32:56 +0200] rev 49712
further support for nested tooltips;
wenzelm [Fri, 05 Oct 2012 13:57:48 +0200] rev 49711
tuned proofs;
wenzelm [Fri, 05 Oct 2012 13:48:22 +0200] rev 49710
refer to parent frame -- relevant for floating dockables in particular;
wenzelm [Fri, 05 Oct 2012 12:11:23 +0200] rev 49709
tuned window position to fit on screen;
wenzelm [Fri, 05 Oct 2012 12:00:28 +0200] rev 49708
tuned window position;
wenzelm [Fri, 05 Oct 2012 11:36:46 +0200] rev 49707
determine window size from content;
wenzelm [Fri, 05 Oct 2012 11:09:24 +0200] rev 49706
tuned color and font size;
wenzelm [Fri, 05 Oct 2012 10:54:07 +0200] rev 49705
close tooltip window on escape;
tuned;
wenzelm [Fri, 05 Oct 2012 10:23:49 +0200] rev 49704
proper message markup for output;
wenzelm [Thu, 04 Oct 2012 20:36:10 +0200] rev 49703
some re-ordering of initialization to ensure proper formatting;
wenzelm [Thu, 04 Oct 2012 20:14:40 +0200] rev 49702
separate module Pretty_Tooltip;
wenzelm [Thu, 04 Oct 2012 19:31:50 +0200] rev 49701
refined rich tooltip options;
basic tooltips without markup;
wenzelm [Thu, 04 Oct 2012 18:28:31 +0200] rev 49700
Rich_Text_Area tooltips via nested Pretty_Text_Area, based on some techniques of FoldViewer plugin;
wenzelm [Thu, 04 Oct 2012 13:56:32 +0200] rev 49699
some documentation of show_markup;
wenzelm [Thu, 04 Oct 2012 11:45:56 +0200] rev 49698
tuned proofs;
wenzelm [Thu, 04 Oct 2012 11:39:24 +0200] rev 49697
option to bypass potentially slow text overview;
wenzelm [Thu, 04 Oct 2012 11:07:36 +0200] rev 49696
tuned signature;
wenzelm [Thu, 04 Oct 2012 10:55:36 +0200] rev 49695
clarified platform dependency;
Gerwin Klein <gerwin.klein@nicta.com.au> [Thu, 04 Oct 2012 09:19:54 +1000] rev 49694
updated crontab and afp-poly settings
blanchet [Wed, 03 Oct 2012 22:07:26 +0200] rev 49693
thread the right local theory through + reenable parallel proofs for previously problematic theories
blanchet [Wed, 03 Oct 2012 21:46:52 +0200] rev 49692
made code more conform to rest of BNF package
wenzelm [Wed, 03 Oct 2012 17:12:08 +0200] rev 49691
more error positions;
wenzelm [Wed, 03 Oct 2012 16:59:58 +0200] rev 49690
more explicit show_type_constraint, show_sort_constraint;
wenzelm [Wed, 03 Oct 2012 16:59:20 +0200] rev 49689
recovered print translation after 'a => bool to 'a set change;
wenzelm [Wed, 03 Oct 2012 16:43:41 +0200] rev 49688
tuned;
wenzelm [Wed, 03 Oct 2012 16:42:36 +0200] rev 49687
use explicit Type.strip_sorts_dummy to suppress sort constraints in output;
wenzelm [Wed, 03 Oct 2012 16:01:07 +0200] rev 49686
printed "_ofsort" is subject to show_markup as well;
wenzelm [Wed, 03 Oct 2012 14:58:56 +0200] rev 49685
allow position constraints to coexist with 0 or 1 sort constraints;
more position information in sorting error;
report sorting of all type variables;
traytel [Tue, 02 Oct 2012 09:20:28 +0200] rev 49684
made tactic more robust (less usage of stac)
blanchet [Tue, 02 Oct 2012 01:00:18 +0200] rev 49683
continued changing type of corec type
blanchet [Tue, 02 Oct 2012 01:00:18 +0200] rev 49682
removed dead params and dead code
blanchet [Tue, 02 Oct 2012 01:00:18 +0200] rev 49681
changed type of corecursor for the nested recursion case
blanchet [Tue, 02 Oct 2012 01:00:18 +0200] rev 49680
made (co)rec tactic more robust when the simplifier succeeds early
wenzelm [Mon, 01 Oct 2012 20:38:57 +0200] rev 49679
tuned;
wenzelm [Mon, 01 Oct 2012 20:35:09 +0200] rev 49678
removed unused module Blob;
wenzelm [Mon, 01 Oct 2012 20:17:30 +0200] rev 49677
more direct message header: eliminated historic encoding via single letter;
wenzelm [Mon, 01 Oct 2012 20:16:37 +0200] rev 49676
tuned whitespace;
wenzelm [Mon, 01 Oct 2012 17:29:00 +0200] rev 49675
tuned proofs;
wenzelm [Mon, 01 Oct 2012 16:37:22 +0200] rev 49674
report sort assignment of visible type variables;
wenzelm [Mon, 01 Oct 2012 12:05:05 +0200] rev 49673
more robust File.eq, and thus File.copy of "~~/lib/logo/isabelle.gif";
blanchet [Mon, 01 Oct 2012 11:04:30 +0200] rev 49672
fixed recursor definition for datatypes with inner products (e.g. "'a trm" from the lambda-term example)
blanchet [Mon, 01 Oct 2012 10:46:30 +0200] rev 49671
tweaked corecursor/coiterator tactic
blanchet [Mon, 01 Oct 2012 10:34:58 +0200] rev 49670
changed the type of the recursor for nested recursion
blanchet [Sun, 30 Sep 2012 23:45:03 +0200] rev 49669
fixed quick-and-dirty mode
blanchet [Sun, 30 Sep 2012 22:02:34 +0200] rev 49668
tuning
traytel [Sun, 30 Sep 2012 12:08:16 +0200] rev 49667
use Thm.close_derivation in theorems proved using Skip_Proof.prove; tuned signature;
traytel [Sun, 30 Sep 2012 12:04:47 +0200] rev 49666
got rid of subst_tac alias
traytel [Sun, 30 Sep 2012 12:04:13 +0200] rev 49665
tuned tactic
wenzelm [Sat, 29 Sep 2012 21:59:08 +0200] rev 49664
tuned proofs;
wenzelm [Sat, 29 Sep 2012 21:24:20 +0200] rev 49663
tuned proofs;
wenzelm [Sat, 29 Sep 2012 20:13:50 +0200] rev 49662
proper handling of constraints stemming from idtyp_ast_tr';
wenzelm [Sat, 29 Sep 2012 19:28:03 +0200] rev 49661
enable show_markup by default (approx. double output size);
wenzelm [Sat, 29 Sep 2012 18:23:46 +0200] rev 49660
more explicit Syntax_Trans.mark_bound_abs/mark_bound_body: preserve type information for show_markup;
wenzelm [Sat, 29 Sep 2012 16:51:04 +0200] rev 49659
explicit show_types takes preferenced over show_markup;
wenzelm [Sat, 29 Sep 2012 16:35:31 +0200] rev 49658
ignore wrapped markup elements in Proof General;
wenzelm [Sat, 29 Sep 2012 16:17:46 +0200] rev 49657
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
proper recursion in standard_format;
wenzelm [Sat, 29 Sep 2012 16:15:18 +0200] rev 49656
treat wrapped markup elements as raw markup delimiters;
wenzelm [Sat, 29 Sep 2012 13:43:23 +0200] rev 49655
tuned signature;
wenzelm [Fri, 28 Sep 2012 23:45:15 +0200] rev 49654
tuned proofs;
wenzelm [Fri, 28 Sep 2012 23:40:48 +0200] rev 49653
tuned proofs;
wenzelm [Fri, 28 Sep 2012 23:02:49 +0200] rev 49652
tuned proofs;
wenzelm [Fri, 28 Sep 2012 23:02:39 +0200] rev 49651
tuned;
wenzelm [Fri, 28 Sep 2012 22:53:18 +0200] rev 49650
support for wrapped XML elements, which allows to preserve full markup tree information in to_XML/from_XML conversion;
wenzelm [Fri, 28 Sep 2012 17:06:07 +0200] rev 49649
merged
wenzelm [Fri, 28 Sep 2012 16:59:53 +0200] rev 49648
eliminated dead code;
wenzelm [Fri, 28 Sep 2012 16:51:58 +0200] rev 49647
smarter handling of tracing messages;
wenzelm [Fri, 28 Sep 2012 15:45:03 +0200] rev 49646
display number of tracing messages;
wenzelm [Fri, 28 Sep 2012 15:25:49 +0200] rev 49645
tuned signature;
wenzelm [Fri, 28 Sep 2012 15:05:16 +0200] rev 49644
tuned proofs;
blanchet [Fri, 28 Sep 2012 15:23:32 +0200] rev 49643
simplified simpset
blanchet [Fri, 28 Sep 2012 15:14:11 +0200] rev 49642
fixed simplification of prod and sum relators to avoid issues with e.g. codata ('a, 'b) k = K "'a + 'b"
traytel [Fri, 28 Sep 2012 13:16:10 +0200] rev 49641
tuned tactic
wenzelm [Fri, 28 Sep 2012 11:46:57 +0200] rev 49640
updated keywords using proper "isabelle update_keywords";
traytel [Fri, 28 Sep 2012 11:31:51 +0200] rev 49639
tuned tactic
traytel [Fri, 28 Sep 2012 09:38:07 +0200] rev 49638
tuned tactic
blanchet [Fri, 28 Sep 2012 09:21:27 +0200] rev 49637
merge
blanchet [Fri, 28 Sep 2012 09:12:50 +0200] rev 49636
renamed ML file in preparation for next step
blanchet [Fri, 28 Sep 2012 09:12:50 +0200] rev 49635
killed temporary "data_raw" and "codata_raw" now that the examples have been ported to "data" and "codata"
blanchet [Fri, 28 Sep 2012 09:12:50 +0200] rev 49634
modernized example, exploiting "rep_compat" option
blanchet [Fri, 28 Sep 2012 09:12:50 +0200] rev 49633
compatibility option to use "rep_datatype"
blanchet [Fri, 28 Sep 2012 09:12:50 +0200] rev 49632
tuned message
blanchet [Fri, 28 Sep 2012 09:12:49 +0200] rev 49631
modernized example
traytel [Fri, 28 Sep 2012 09:17:30 +0200] rev 49630
tuned tactics
nipkow [Fri, 28 Sep 2012 08:59:54 +0200] rev 49629
second usage of const_typ
nipkow [Fri, 28 Sep 2012 08:39:48 +0200] rev 49628
new antiquotation const_typ
nipkow [Fri, 28 Sep 2012 08:09:28 +0200] rev 49627
tuned printing of _ in latex
kuncar [Thu, 27 Sep 2012 20:30:32 +0200] rev 49626
mk_readable_rsp_thm_eq is more robust now
kuncar [Thu, 27 Sep 2012 20:30:30 +0200] rev 49625
new get function for non-symmetric relator_eq & tuned
wenzelm [Thu, 27 Sep 2012 19:35:29 +0200] rev 49624
merged
traytel [Thu, 27 Sep 2012 18:58:15 +0200] rev 49623
tuned tactic; got rid of substs_tac alias
blanchet [Thu, 27 Sep 2012 18:39:17 +0200] rev 49622
use a nicer scheme to indexify names
traytel [Thu, 27 Sep 2012 18:25:41 +0200] rev 49621
tuned tactic
traytel [Thu, 27 Sep 2012 18:01:33 +0200] rev 49620
type of the bound of a BNF depends at most on dead type variables
blanchet [Thu, 27 Sep 2012 17:54:35 +0200] rev 49619
repaired signature
blanchet [Thu, 27 Sep 2012 17:00:54 +0200] rev 49618
lower the defaults for the number of bits, based on an example by Lukas Bulwahn
blanchet [Thu, 27 Sep 2012 17:00:54 +0200] rev 49617
modernized examples
nipkow [Thu, 27 Sep 2012 12:08:38 +0200] rev 49616
merged
nipkow [Thu, 27 Sep 2012 12:07:50 +0200] rev 49615
tuned
wenzelm [Thu, 27 Sep 2012 19:34:31 +0200] rev 49614
operations to turn markup into XML;
tuned;
wenzelm [Thu, 27 Sep 2012 15:55:38 +0200] rev 49613
removed obsolete org.w3c.dom operations;
wenzelm [Thu, 27 Sep 2012 15:38:28 +0200] rev 49612
eliminated obsolete HTML/CSS functionality;
wenzelm [Thu, 27 Sep 2012 15:09:32 +0200] rev 49611
removed obsolete Output1 dockable;
wenzelm [Thu, 27 Sep 2012 15:04:26 +0200] rev 49610
physical File.eq in conformance to Isabelle/ML;
wenzelm [Thu, 27 Sep 2012 14:52:50 +0200] rev 49609
tuned proofs;
wenzelm [Thu, 27 Sep 2012 14:50:06 +0200] rev 49608
tuned;
wenzelm [Thu, 27 Sep 2012 14:46:34 +0200] rev 49607
updated to consolidated SortedMap in scala-2.9.x;
blanchet [Thu, 27 Sep 2012 10:59:10 +0200] rev 49606
partly ported "TreeFI" example to new syntax
blanchet [Thu, 27 Sep 2012 10:59:10 +0200] rev 49605
avoid another brand of trivial "disc_rel" theorems (which made the simplifier loop for all single-constructor types)
nipkow [Thu, 27 Sep 2012 10:43:40 +0200] rev 49604
tuned
nipkow [Thu, 27 Sep 2012 10:20:38 +0200] rev 49603
tuned
blanchet [Thu, 27 Sep 2012 00:41:08 +0200] rev 49602
merge
blanchet [Thu, 27 Sep 2012 00:40:51 +0200] rev 49601
modernized examples;
removed now trivial "HFset"
wenzelm [Wed, 26 Sep 2012 23:30:19 +0200] rev 49600
some support for jEdit warmstart;
wenzelm [Wed, 26 Sep 2012 19:50:10 +0200] rev 49599
discontinued XML.cache experiment -- Poly/ML 5.5.0 RTS does online sharing better;
wenzelm [Wed, 26 Sep 2012 16:37:21 +0200] rev 49598
tuned message;
wenzelm [Wed, 26 Sep 2012 15:04:15 +0200] rev 49597
merged
blanchet [Wed, 26 Sep 2012 10:41:36 +0200] rev 49596
disable parallel proofs for two big examples -- speeds up things and eliminates spurious Interrupt exceptions (to be investigated)
blanchet [Wed, 26 Sep 2012 10:01:00 +0200] rev 49595
got rid of other instance of shaky "Thm.generalize"
blanchet [Wed, 26 Sep 2012 10:01:00 +0200] rev 49594
tweaked theorem names (in particular, dropped s's)
blanchet [Wed, 26 Sep 2012 10:01:00 +0200] rev 49593
get rid of shaky "Thm.generalize"
blanchet [Wed, 26 Sep 2012 10:01:00 +0200] rev 49592
fixed "rels" + split them into injectivity and distinctness
blanchet [Wed, 26 Sep 2012 10:00:59 +0200] rev 49591
generate high-level "coinduct" and "strong_coinduct" properties
blanchet [Wed, 26 Sep 2012 10:00:59 +0200] rev 49590
added coinduction tactic
blanchet [Wed, 26 Sep 2012 10:00:59 +0200] rev 49589
generalized tactic a bit
blanchet [Wed, 26 Sep 2012 10:00:59 +0200] rev 49588
export "dtor_map_coinduct" theorems, since they're used in one example
blanchet [Wed, 26 Sep 2012 10:00:59 +0200] rev 49587
name tuning
blanchet [Wed, 26 Sep 2012 10:00:59 +0200] rev 49586
parameterized "subst_tac"
blanchet [Wed, 26 Sep 2012 10:00:59 +0200] rev 49585
generate high-level "maps", "sets", and "rels" properties
blanchet [Wed, 26 Sep 2012 10:00:59 +0200] rev 49584
use singular since there is always only one theorem
blanchet [Wed, 26 Sep 2012 10:00:59 +0200] rev 49583
nicer type var names
blanchet [Wed, 26 Sep 2012 10:00:59 +0200] rev 49582
renamed "dtor_rel_coinduct" etc. to "dtor_coinduct"
blanchet [Wed, 26 Sep 2012 10:00:59 +0200] rev 49581
renamed "dtor_coinduct" etc. to "dtor_map_coinduct"
blanchet [Wed, 26 Sep 2012 10:00:59 +0200] rev 49580
leave out some internal theorems unless "bnf_note_all" is set
nipkow [Wed, 26 Sep 2012 03:16:40 +0200] rev 49579
tuned
nipkow [Wed, 26 Sep 2012 03:03:11 +0200] rev 49578
added counterexamples
nipkow [Wed, 26 Sep 2012 02:51:59 +0200] rev 49577
tuned
nipkow [Tue, 25 Sep 2012 07:37:42 +0200] rev 49576
tuned
wenzelm [Wed, 26 Sep 2012 15:01:45 +0200] rev 49575
more uniform graphview terminology;
wenzelm [Wed, 26 Sep 2012 14:56:59 +0200] rev 49574
proper Symbol.decode -- especially relevant for Proof General;
wenzelm [Wed, 26 Sep 2012 14:55:51 +0200] rev 49573
suppress empty tooltips;
wenzelm [Wed, 26 Sep 2012 14:52:18 +0200] rev 49572
obsolete;
wenzelm [Wed, 26 Sep 2012 14:50:46 +0200] rev 49571
updated keywords;
wenzelm [Wed, 26 Sep 2012 14:38:23 +0200] rev 49570
more uniform graphview terminology;
wenzelm [Wed, 26 Sep 2012 14:23:33 +0200] rev 49569
tuned pretty_locale/print_locale, with more basic pretty_locale_deps based on that;
added command 'locale_deps';
graphview prints plain text only -- removed dependency on old Cobra HTML_Panel;
wenzelm [Wed, 26 Sep 2012 14:13:07 +0200] rev 49568
proper install_fonts;
wenzelm [Tue, 25 Sep 2012 22:52:40 +0200] rev 49567
proper jvmpath for Windows;
wenzelm [Tue, 25 Sep 2012 22:36:06 +0200] rev 49566
basic integration of graphview into document model;
added Graph_Dockable;
updated Isabelle/jEdit authors and dependencies etc.;
wenzelm [Tue, 25 Sep 2012 20:28:47 +0200] rev 49565
ML support for generic graph display, with browser and graphview backends (via print modes);
reverse graph layout (again), according to the graph orientation provided by ML;
simplified scala types -- eliminated unused type parameters;
more explicit Model.Info, Model.Graph;
renamed isabelle.graphview.Graphview_Frame to isabelle.graphview.Frame in accordance to file name;
removed obsolete Graph_XML and Tooltips;
tuned graphview command line;
more generous JVM resources via GRAPHVIEW_JAVA_OPTIONS;
wenzelm [Tue, 25 Sep 2012 18:24:49 +0200] rev 49564
tuned;
wenzelm [Tue, 25 Sep 2012 16:55:32 +0200] rev 49563
more complete build;
added option -c to imitate old browser;
wenzelm [Tue, 25 Sep 2012 16:48:33 +0200] rev 49562
proper error message;
wenzelm [Tue, 25 Sep 2012 15:40:41 +0200] rev 49561
separate module Graph_Display;
tuned signature;
wenzelm [Tue, 25 Sep 2012 14:32:41 +0200] rev 49560
added graph encode/decode operations;
tuned signature;
wenzelm [Tue, 25 Sep 2012 12:17:58 +0200] rev 49559
tuned;
wenzelm [Mon, 24 Sep 2012 21:16:33 +0200] rev 49558
minimal component and build setup for graphview;
Markus Kaiser <markus.kaiser@in.tum.de> [Mon, 24 Sep 2012 20:22:58 +0200] rev 49557
added Graphview tool, based on Isabelle/Scala and Swing/Graphics2D;
haftmann [Mon, 24 Sep 2012 19:11:35 +0200] rev 49556
made smlnj even happier
wenzelm [Mon, 24 Sep 2012 17:52:44 +0200] rev 49555
tuned proofs;
wenzelm [Mon, 24 Sep 2012 17:28:36 +0200] rev 49554
more explicit keyword1/keyword2 markup -- avoid potential conflict with input token markup produced by Token_Marker;
wenzelm [Mon, 24 Sep 2012 16:41:51 +0200] rev 49553
updated checksum, which appears to have changed accidentally;
wenzelm [Mon, 24 Sep 2012 16:39:26 +0200] rev 49552
updated to exec_process-1.0.2;
wenzelm [Mon, 24 Sep 2012 16:27:48 +0200] rev 49551
search bash via PATH as usual (this is no longer restricted to Cygwin with its known file-system layout);
wenzelm [Mon, 24 Sep 2012 16:13:56 +0200] rev 49550
discontinued futile attempt to hardwire build options into the image, sequential mode is enabled more robustly at runtime (cf. 3b0a60eee56e);
wenzelm [Mon, 24 Sep 2012 15:37:58 +0200] rev 49549
Mirabelle appears to work better in single-threaded mode;
nipkow [Mon, 24 Sep 2012 14:22:07 +0200] rev 49548
generalized types
nipkow [Mon, 24 Sep 2012 06:58:09 +0200] rev 49547
tuned termination proof
blanchet [Sun, 23 Sep 2012 14:52:53 +0200] rev 49546
adapted examples to new names
blanchet [Sun, 23 Sep 2012 14:52:53 +0200] rev 49545
renamed coinduction principles to have "dtor" in the name
blanchet [Sun, 23 Sep 2012 14:52:53 +0200] rev 49544
renamed "set_incl" etc. to have "ctor" or "dtor" in the name
blanchet [Sun, 23 Sep 2012 14:52:53 +0200] rev 49543
renamed low-level "map_unique" to have "ctor" or "dtor" in the name
blanchet [Sun, 23 Sep 2012 14:52:53 +0200] rev 49542
renamed low-level "set_simps" and "set_induct" to have "ctor" or "dtor" in the name
blanchet [Sun, 23 Sep 2012 14:52:53 +0200] rev 49541
renamed "map_simps" to "{c,d}tor_maps"
blanchet [Sun, 23 Sep 2012 14:52:53 +0200] rev 49540
took out accidentally submitted "tracing" calls
blanchet [Sun, 23 Sep 2012 14:52:53 +0200] rev 49539
fixed bug in "fold" tactic with nested products (beyond the sum of product corresponding to constructors)
blanchet [Sun, 23 Sep 2012 14:52:53 +0200] rev 49538
simplified fact policies
blanchet [Sun, 23 Sep 2012 14:52:53 +0200] rev 49537
generate "rel_as_srel" and "rel_flip" properties
blanchet [Sun, 23 Sep 2012 14:52:53 +0200] rev 49536
started work on generation of "rel" theorems
haftmann [Sun, 23 Sep 2012 08:24:19 +0200] rev 49535
make smlnj happy
haftmann [Sat, 22 Sep 2012 21:59:40 +0200] rev 49534
more strict typscheme_equiv check: must fix variables of more specific type;
dropped dead code;
tuned order
haftmann [Sat, 22 Sep 2012 21:59:40 +0200] rev 49533
cache should not contain material from descendant theory
wenzelm [Sat, 22 Sep 2012 21:23:16 +0200] rev 49532
some PIDE NEWS from this summer;
wenzelm [Sat, 22 Sep 2012 20:38:42 +0200] rev 49531
tuned whitespace;
wenzelm [Sat, 22 Sep 2012 20:37:47 +0200] rev 49530
tuned;
wenzelm [Sat, 22 Sep 2012 20:29:28 +0200] rev 49529
tuned proofs;
wenzelm [Sat, 22 Sep 2012 19:32:30 +0200] rev 49528
report proper binding positions only -- avoid swamping document model with unspecific information;
wenzelm [Sat, 22 Sep 2012 19:23:04 +0200] rev 49527
accumulate under exec_id as well;
wenzelm [Sat, 22 Sep 2012 19:16:48 +0200] rev 49526
more restrictive pattern, to avoid malformed positions intruding the command range (cf. d7a1973b063c);
wenzelm [Sat, 22 Sep 2012 17:55:56 +0200] rev 49525
misc tuning;
wenzelm [Sat, 22 Sep 2012 14:41:41 +0200] rev 49524
Thy_Syntax.consolidate_spans is subject to editor_reparse_limit, for improved experience of unbalanced comments etc.;
wenzelm [Sat, 22 Sep 2012 14:03:01 +0200] rev 49523
tuned signature;
wenzelm [Fri, 21 Sep 2012 22:45:14 +0200] rev 49522
tuned proofs;
wenzelm [Fri, 21 Sep 2012 21:24:48 +0200] rev 49521
misc tuning;
wenzelm [Fri, 21 Sep 2012 21:24:33 +0200] rev 49520
tighten margin for TextArea instead of Lobo;
wenzelm [Fri, 21 Sep 2012 20:54:48 +0200] rev 49519
misc tuning;
blanchet [Fri, 21 Sep 2012 19:17:49 +0200] rev 49518
renamed LFP low-level rel property to have ctor not dtor in its name
blanchet [Fri, 21 Sep 2012 18:25:17 +0200] rev 49517
changed base session for "HOL-BNF" for faster building in the typical case
blanchet [Fri, 21 Sep 2012 18:25:17 +0200] rev 49516
renamed "rel_simp" to "dtor_rel" and similarly for "srel"
blanchet [Fri, 21 Sep 2012 18:25:17 +0200] rev 49515
fixed a few names that escaped the renaming
blanchet [Fri, 21 Sep 2012 18:25:17 +0200] rev 49514
tuned whitespace