Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
VCG is standard name
2013-05-31, by nipkow
used nice syntax, removed lemma because it makes a nice exercise.
2013-05-31, by nipkow
NEWS about Spec_Check
2013-05-31, by bulwahn
tuned headers;
2013-05-30, by wenzelm
tuned messages -- some attempts to observe Isabelle output channel semantics;
2013-05-30, by wenzelm
less verbosity -- do not print final ();
2013-05-30, by wenzelm
tuned -- dynamic ML context is updated incrementally (see also e7c47fe56fbd);
2013-05-30, by wenzelm
tuned;
2013-05-30, by wenzelm
toplevel invocation via implicit ML compilation context;
2013-05-30, by wenzelm
more direct Context.setmp_thread_data for one-way passing of context;
2013-05-30, by wenzelm
tuned;
2013-05-30, by wenzelm
tuned;
2013-05-30, by wenzelm
do not open ML structures;
2013-05-30, by wenzelm
prefer separate 'ML_command' for parallel evaluation;
2013-05-30, by wenzelm
simplified context and data management -- plain ctxt: Proof.context is default for most operations;
2013-05-30, by wenzelm
more conventional spelling and grammar;
2013-05-30, by wenzelm
minor tuning -- more linebreaks;
2013-05-30, by wenzelm
removed pointless comment -- NB: Isabelle output is message-oriented with implicit line-boundaries;
2013-05-30, by wenzelm
standardized aliases;
2013-05-30, by wenzelm
do not handle arbitrary exceptions;
2013-05-30, by wenzelm
added Spec_Check -- a Quickcheck tool for Isabelle's ML environment;
2013-05-30, by bulwahn
merged
2013-05-30, by wenzelm
tuned signature;
2013-05-30, by wenzelm
tuned signature;
2013-05-30, by wenzelm
misc tuning;
2013-05-30, by wenzelm
prefer existing beta_eta_conversion;
2013-05-30, by wenzelm
more standard fold/fold_rev;
2013-05-30, by wenzelm
tuned import;
2013-05-30, by wenzelm
misc tuning;
2013-05-30, by wenzelm
prefer existing beta_eta_conversion;
2013-05-30, by wenzelm
more standard names;
2013-05-30, by wenzelm
simplified method setup;
2013-05-30, by wenzelm
tuned -- prefer terminology of tactic / goal state;
2013-05-30, by wenzelm
tuned;
2013-05-30, by wenzelm
misc tuning;
2013-05-30, by wenzelm
tuned;
2013-05-30, by wenzelm
tuned signature;
2013-05-30, by wenzelm
stay within regular tactic language -- avoid operating on whole proof state;
2013-05-30, by wenzelm
standardized aliases;
2013-05-30, by wenzelm
space between minus sign and number for large negative number literals causes NumberFormatException at run-time
2013-05-30, by Andreas Lochbihler
tuned
2013-05-30, by nipkow
relational version of HoareT
2013-05-30, by kleing
obsolete;
2013-05-29, by wenzelm
resolve_inc_tyvars: back to old behavior before 0fa3b456a267 where types of equal Vars are *not* unified -- recover last example in src/HOL/Metis_Examples/Clausification.thy;
2013-05-29, by wenzelm
more precise "incremented" indication, which might be relevant in corner cases, e.g. instantiation of leading to vars with different types (which is a potential problem nonetheless);
2013-05-29, by wenzelm
tuned signature -- more explicit flags for low-level Thm.bicompose;
2013-05-29, by wenzelm
unify types of schematic variables in non-lifted case (i.e. "compose variants") -- allow schematic polymorphism, without revisiting HO-unification;
2013-05-29, by wenzelm
tuned signature;
2013-05-29, by wenzelm
backout 3b9c31867707 -- too risky to "amend" modules from 25 years ago that don't handle Vars with different types;
2013-05-29, by wenzelm
observe type annotations in print translations as well, notably type_constraint_tr';
2013-05-29, by wenzelm
make SML/NJ happy;
2013-05-29, by wenzelm
tuning
2013-05-29, by blanchet
more work on general recursors
2013-05-29, by blanchet
tuning (use lists rather than pairs of lists throughout)
2013-05-29, by blanchet
generalized recursors, effectively reverting inductive half of c7a034d01936
2013-05-29, by blanchet
tuning
2013-05-29, by blanchet
merged
2013-05-28, by wenzelm
explicit support for type annotations within printed syntax trees;
2013-05-28, by wenzelm
more explicit Printer.type_emphasis, depending on show_type_emphasis;
2013-05-28, by wenzelm
tuning (refactoring)
2013-05-28, by blanchet
refactored triplicated functionality
2013-05-28, by blanchet
tuning -- avoided unreadable true/false all over the place for LFP/GFP
2013-05-28, by blanchet
merge
2013-05-28, by blanchet
don't create needless constant
2013-05-28, by blanchet
merged
2013-05-28, by popescua
fixed broken Cardinals and BNF due to Order_Union
2013-05-28, by popescua
no confusing special behavior in debug mode
2013-05-28, by blanchet
tuned Nitpick message to be in sync with similar warning from Kodkod
2013-05-28, by blanchet
merged
2013-05-28, by popescua
merged Well_Order_Extension into Zorn
2013-05-28, by popescua
removed junk (cf. 667961fa6a60);
2013-05-28, by wenzelm
exported ML function
2013-05-28, by blanchet
redid rac7830871177 to avoid duplicate fixed variable (e.g. lemma "P (a::nat)" proof - have "!!a::int. Q a" sledgehammer [e])
2013-05-28, by blanchet
clean up list of theorems
2013-05-28, by blanchet
removed needless comment (yes, sum_case_if is needed)
2013-05-28, by blanchet
tuned
2013-05-28, by nipkow
actually test theory Order_Union;
2013-05-27, by wenzelm
more direct notation;
2013-05-27, by wenzelm
merged
2013-05-27, by wenzelm
more literal tokens, e.g. "EX!";
2013-05-27, by wenzelm
report markup for ast translations;
2013-05-27, by wenzelm
tuned;
2013-05-27, by wenzelm
tuned;
2013-05-27, by wenzelm
discontinued obsolete show_all_types;
2013-05-27, by wenzelm
added Ordered_Union
2013-05-27, by popescua
fixed files broken due to Zorn changes (cf. 59e5dd7b8f9a)
2013-05-24, by popescua
well-order extension (by Christian Sternagel)
2013-05-24, by popescua
modernized Zorn (by Christian Sternagel)
2013-05-24, by popescua
merged
2013-05-27, by wenzelm
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
2013-05-27, by wenzelm
instantiate types as well (see also Thm.first_order_match);
2013-05-27, by wenzelm
tuned;
2013-05-27, by wenzelm
updated to ProofGeneral-4.2;
2013-05-27, by wenzelm
uniform Term_Position.markers (cf. dbadb4d03cbc);
2013-05-27, by wenzelm
get rid of "show_all_types" in Nitpick
2013-05-27, by blanchet
tuning
2013-05-27, by blanchet
killed dead argument
2013-05-27, by blanchet
tuning
2013-05-27, by blanchet
generalized "mk_co_iter" to handle mutualized (co)iterators
2013-05-27, by blanchet
tuning
2013-05-27, by blanchet
tuned
2013-05-27, by nipkow
tuned
2013-05-27, by nipkow
merged
2013-05-27, by nipkow
tuned
2013-05-27, by nipkow
merged
2013-05-26, by wenzelm
position constraint for bound dummy -- more PIDE markup;
2013-05-26, by wenzelm
position constraint for dummy_pattern -- more PIDE markup;
2013-05-26, by wenzelm
tuned;
2013-05-26, by wenzelm
tuned signature;
2013-05-26, by wenzelm
tuned -- less ML compiler warnings;
2013-05-26, by wenzelm
more robust variant_free: avoid clash with consts name space (e.g. consts "x", "xa", etc.);
2013-05-26, by wenzelm
more uniform context;
2013-05-26, by wenzelm
tuned signature;
2013-05-26, by wenzelm
more conventional pretty printing;
2013-05-26, by wenzelm
tuned white-space;
2013-05-26, by wenzelm
more specific structure for registration into theory and dependency onto locale
2013-05-26, by haftmann
examples for interpretation into target
2013-05-26, by haftmann
disable SPASS's splitting if Isar proofs are desired, because these are not handled by the proof reconstruction code (and it's not clear how to handle them considering the lack of documentation)
2013-05-26, by blanchet
handle lambda-lifted problems in Isar construction code
2013-05-26, by blanchet
simpler proof through custom summation function
2013-05-26, by nipkow
merged
2013-05-25, by wenzelm
tuned;
2013-05-25, by wenzelm
tuned;
2013-05-25, by wenzelm
tuned;
2013-05-25, by wenzelm
tuned;
2013-05-25, by wenzelm
syntax translations always depend on context;
2013-05-25, by wenzelm
updated keywords;
2013-05-25, by wenzelm
weaker precendence of syntax for big intersection and union on sets
2013-05-25, by haftmann
tuned structure
2013-05-25, by haftmann
add lemma
2013-05-25, by noschinl
bookkeeping and input syntax for exact specification of names of symbols in generated code
2013-05-24, by haftmann
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
2013-05-24, by haftmann
dedicated module for code symbol data
2013-05-24, by haftmann
symbol data covers class relations also
2013-05-24, by haftmann
merged
2013-05-24, by wenzelm
proper internal error, not user error;
2013-05-24, by wenzelm
tuned;
2013-05-24, by wenzelm
tuned signature;
2013-05-24, by wenzelm
tuned;
2013-05-24, by wenzelm
unify types of bound variables in the same manner as Unify.new_dpair (which emphatically "Tries to unify types of the bound variables!");
2013-05-24, by wenzelm
tuned signature -- slightly more general operations (cf. term.ML);
2013-05-24, by wenzelm
re-use Pattern.unify_types, including its trace_unify_fail option;
2013-05-24, by wenzelm
tuned signature;
2013-05-24, by wenzelm
improved handling of free variables' types in Isar proofs
2013-05-24, by blanchet
pass noninteractive flag -- necessary to run under CASC's "runsolver" program
2013-05-24, by blanchet
untabify
2013-05-24, by blanchet
more lemmas for sorted_list_of_set
2013-05-23, by noschinl
prefer object equality
2013-05-23, by kleing
slightly clearer formulation
2013-05-23, by kleing
interpretation must always operate on the last element in a local theory stack, not on all elements: interpretated facts must disappear after pop from local theory stack, and transfer from last target is not enough
2013-05-22, by haftmann
mark local theory as brittle also after interpretation inside locales;
2013-05-22, by haftmann
merged
2013-05-22, by wenzelm
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
2013-05-22, by wenzelm
tuned signature;
2013-05-22, by wenzelm
more informative Build.build_results;
2013-05-22, by wenzelm
stop protocol handlers as well;
2013-05-22, by wenzelm
more robust command line -- accomodate /bin/kill on recent Linux (e.g. Xubuntu 13.04):
2013-05-22, by wenzelm
explicit management of Session.Protocol_Handlers, with protocol state and functions;
2013-05-22, by wenzelm
prevent pretty printer from automatically annotating numerals
2013-05-22, by smolkas
tuned
2013-05-22, by smolkas
simplified example and proof
2013-05-22, by nipkow
tuned
2013-05-22, by nipkow
tuned messages;
2013-05-21, by wenzelm
proper options;
2013-05-21, by wenzelm
proper options;
2013-05-21, by wenzelm
more markup;
2013-05-21, by wenzelm
tuned;
2013-05-21, by wenzelm
less intrusive rendering of antiquoted text -- avoid visual clash with "blue variables" in particular;
2013-05-21, by wenzelm
proper context;
2013-05-21, by wenzelm
make SML/NJ happy;
2013-05-21, by wenzelm
added CASC-related files, to keep a public record of the Isabelle submission at the competition
2013-05-21, by blanchet
disabled choice in Satallax
2013-05-21, by blanchet
use HOL-TPTP image in TPTP tools (for less verbose and faster startup) and filter out some messages
2013-05-21, by blanchet
prefer compiled version of LEO-II and Satallax if available
2013-05-21, by blanchet
updated remote provers
2013-05-21, by blanchet
added compatibility alias
2013-05-21, by blanchet
merged
2013-05-20, by wenzelm
more rigorous check of simplifier context;
2013-05-20, by wenzelm
proper context;
2013-05-20, by wenzelm
proper context;
2013-05-20, by wenzelm
proper run-time context;
2013-05-20, by wenzelm
more precise treatment of theory vs. Proof.context;
2013-05-20, by wenzelm
proper run-time context;
2013-05-20, by wenzelm
tuned;
2013-05-20, by wenzelm
more explicit Session.update_options as source of Global_Options event;
2013-05-20, by wenzelm
even later Options.reset_default -- still needed for printing errors of Session.finish (e.g. via Command_Line.tool0);
2013-05-20, by wenzelm
tuned;
2013-05-20, by wenzelm
discontinued odd workaround for scala-2.9.2, which is hopefully obsolete in scala-2.10.x;
2013-05-20, by wenzelm
reset options last -- other parts of the system may still need them;
2013-05-20, by wenzelm
tuned signature;
2013-05-20, by wenzelm
updated Sledgehammer docs
2013-05-20, by blanchet
parse agsyHOL proofs (as unsat cores)
2013-05-20, by blanchet
freeze types in Sledgehammer goal, not just terms
2013-05-20, by blanchet
generate agsyHOL-friendly THF (to some extent -- partial application of connectives remains an issue)
2013-05-20, by blanchet
tuned code
2013-05-20, by blanchet
started adding agsyHOL as an experimental prover
2013-05-20, by blanchet
defined lvars and rvars of commands separately.
2013-05-20, by nipkow
made "completish" mode a bit more complete
2013-05-19, by blanchet
infrastructure for generic data for code symbols (constants, type constructors, classes, instances)
2013-05-19, by haftmann
tuned and clarified
2013-05-19, by haftmann
tuned, including signature
2013-05-19, by haftmann
discontinued odd workaround for scala-2.10.0-RC1;
2013-05-18, by wenzelm
discontinued odd workaround for scala-2.9.2, which is hopefully obsolete in scala-2.10.x;
2013-05-18, by wenzelm
explicit notion of public options, which are shown in the editor options dialog;
2013-05-18, by wenzelm
back to more paranoid interrupt test after request is cancelled -- avoid race condition;
2013-05-17, by wenzelm
timeout counts as regular error, with rc = 1 (cf. special Exn.Interrupt vs. regular TimeLimit.TimeOut in Isabelle/ML);
2013-05-17, by wenzelm
added isabelle tty option -o;
2013-05-17, by wenzelm
oops;
2013-05-17, by wenzelm
renamed 'print_configs' to 'print_options';
2013-05-17, by wenzelm
proper option quick_and_dirty;
2013-05-17, by wenzelm
retain quick_and_dirty as-is -- no censorship;
2013-05-17, by wenzelm
more system-atic options;
2013-05-17, by wenzelm
added isabelle-process option -o;
2013-05-17, by wenzelm
more precise "eval", cf. isabelle build;
2013-05-17, by wenzelm
discontinued obsolete isabelle-process options -f and -u;
2013-05-17, by wenzelm
NEWS;
2013-05-17, by wenzelm
discontinued obsolete isabelle usedir, mkdir, make;
2013-05-17, by wenzelm
modernized TimeLimit.timeLimit using Event_Timer service -- based on more elementary version 11ae688e4e30;
2013-05-17, by wenzelm
event timer as separate service thread;
2013-05-17, by wenzelm
tuned signature;
2013-05-17, by wenzelm
tuned signature -- emphasize thread creation here;
2013-05-17, by wenzelm
repair after bc01725d7918;
2013-05-17, by wenzelm
replaced `;' by `;;' to disambiguate syntax; unexpected slight increase in build time
2013-05-17, by nipkow
tuned
2013-05-17, by nipkow
merged
2013-05-16, by wenzelm
more system options as context-sensitive config options;
2013-05-16, by wenzelm
Thy_Output.modes as proper option;
2013-05-16, by wenzelm
some system options as context-sensitive config options;
2013-05-16, by wenzelm
system options as context-sensitive configuration options within the attribute name space;
2013-05-16, by wenzelm
tuned signature;
2013-05-16, by wenzelm
properly handle SPASS constructors w.r.t. partially applied functions
2013-05-16, by blanchet
tuned signature -- depend on context by default;
2013-05-16, by wenzelm
reflexivity rules for the function type and equality
2013-05-16, by kuncar
tuned comments
2013-05-16, by blanchet
correctly 'repair' the monomorphization context for SMT solvers from Sledgehammer
2013-05-16, by blanchet
tuning
2013-05-16, by blanchet
more work on SPASS datatypes
2013-05-16, by blanchet
tuning -- renamed '_from_' to '_of_' in Sledgehammer
2013-05-16, by blanchet
compile
2013-05-16, by blanchet
don't recognize overloaded constants as constructors for the purpose of removing type arguments
2013-05-16, by blanchet
tuning
2013-05-16, by blanchet
reintroduced syntax for "nonexhaustive" datatypes
2013-05-16, by blanchet
tuning
2013-05-16, by blanchet
more work on SPASS datatypes
2013-05-16, by blanchet
merged
2013-05-16, by Andreas Lochbihler
setup for set membership as a predicate for code_pred
2013-05-16, by Andreas Lochbihler
tuned
2013-05-16, by nipkow
explicitly state equivalence relation for sim; tweak syntax of sem_equiv
2013-05-16, by kleing
merged
2013-05-16, by nipkow
finally: acom with pointwise access and update of annotations
2013-05-16, by nipkow
merged;
2013-05-15, by wenzelm
clarified preferences: "override" re-initialized on prover startup, and "default" sent to PG -- thus recover typical defaults like auto-quickcheck in PG 4.x;
2013-05-15, by wenzelm
simplified ProofGeneral.preference operation -- no need for CRITICAL section for atomic access (and sequential execution of PG/TTY loop);
2013-05-15, by wenzelm
back to hidden welcome -- revert change 9ebf2da69b29, which appears to disturb startup protocol of PG 4.1;
2013-05-15, by wenzelm
more standard Isabelle/ML structures for global preferences;
2013-05-15, by wenzelm
more basic print mode "ProofGeneral" (again);
2013-05-15, by wenzelm
uniform welcome -- actually visible on startup via Output.urgent_message;
2013-05-15, by wenzelm
more elementary ProofGeneral.thm_deps;
2013-05-15, by wenzelm
tuned;
2013-05-15, by wenzelm
moved files;
2013-05-15, by wenzelm
clarified default for Proofterm.proofs, according to etc/options and innermost setmp;
2013-05-15, by wenzelm
maintain ProofGeneral preferences within ProofGeneral module;
2013-05-15, by wenzelm
just one ProofGeneral module;
2013-05-15, by wenzelm
tuning
2013-05-15, by blanchet
more work on SPASS datatypes
2013-05-15, by blanchet
tuning
2013-05-15, by blanchet
no need to reinvent the wheel ("fold_map")
2013-05-15, by blanchet
more work on implementing datatype output for new SPASS
2013-05-15, by blanchet
tuned code
2013-05-15, by blanchet
compile
2013-05-15, by blanchet
renamed Sledgehammer functions with 'for' in their names to 'of'
2013-05-15, by blanchet
added datatype declaration syntax for next-gen SPASS
2013-05-15, by blanchet
abstract equalities only in a correspondence relation in a transfer domain rule
2013-05-15, by kuncar
superfluous transfer rule
2013-05-15, by kuncar
stronger reflexivity prover
2013-05-15, by kuncar
simplified modules and exceptions;
2013-05-14, by wenzelm
more elementary pgiptype;
2013-05-14, by wenzelm
prefer Markup.parse/print operations -- slight change of exception behaviour;
2013-05-14, by wenzelm
more uniform Markup.print_real;
2013-05-14, by wenzelm
removed dead code;
2013-05-14, by wenzelm
more uniform Markup.parse_real;
2013-05-14, by wenzelm
tuned signature;
2013-05-14, by wenzelm
more robust load_timings: ignore JVM errors such as java.lang.OutOfMemoryError;
2013-05-14, by wenzelm
tuned;
2013-05-14, by wenzelm
misc tuning and simplification;
2013-05-14, by wenzelm
more frugal line termination, to cope with huge log files (see also 016cb7d8f297);
2013-05-14, by wenzelm
more scalable File.write via separate chunks;
2013-05-14, by wenzelm
more scalable Library.separate -- NB: JVM has tiny fixed-size stack;
2013-05-14, by wenzelm
support for more informative crashes;
2013-05-14, by wenzelm
more antiquotations;
2013-05-14, by wenzelm
tuned messages;
2013-05-14, by wenzelm
more generous java resources via ISABELLE_BUILD_JAVA_OPTIONS;
2013-05-14, by wenzelm
generate valid direct Isar proof also if the facts are contradictory
2013-05-14, by blanchet
tuned names
2013-05-14, by nipkow
tuned names
2013-05-14, by nipkow
removed obsolete PGIP material;
2013-05-13, by wenzelm
more direct output of remaining PGIP rudiments;
2013-05-13, by wenzelm
simplified preferences, removed obsolete operations;
2013-05-13, by wenzelm
tuned signature;
2013-05-13, by wenzelm
more direct output of remaining PGIP rudiments;
2013-05-13, by wenzelm
obsolete;
2013-05-13, by wenzelm
removed obsolete PGIP material;
2013-05-13, by wenzelm
recovered informative progress from 016cb7d8f297;
2013-05-13, by wenzelm
removed obsolete PGIP material;
2013-05-13, by wenzelm
clean startup of RAW session;
2013-05-13, by wenzelm
dummy PGIP id, which appears to be sufficient for PG/Emacs;
2013-05-13, by wenzelm
limit build process output, to avoid bombing Isabelle/Scala process by ill-behaved jobs (e.g. Containers in AFP/9025435b29cf);
2013-05-13, by wenzelm
merged
2013-05-13, by wenzelm
option "goals_limit", with more uniform description;
2013-05-13, by wenzelm
clarified message when subgoals have been stripped -- unconditional;
2013-05-13, by wenzelm
retain goal display options when printing error messages, to avoid breakdown for huge goals;
2013-05-13, by wenzelm
typo
2013-05-13, by kuncar
better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
2013-05-13, by kuncar
try to detect assumptions of transfer rules that are in a shape of a transfer rule
2013-05-13, by kuncar
publish a private function
2013-05-13, by kuncar
tuned names
2013-05-13, by nipkow
re-init ISABELLE_PROCESS_OPTIONS to allow nested ISABELLE_PROCESS invocations, e.g. HOL-Mutabelle-ex;
2013-05-12, by wenzelm
more standard Isabelle/ML operations -- avoid inaccurate Bool.fromString;
2013-05-12, by wenzelm
prefer standard Isabelle/ML operations;
2013-05-12, by wenzelm
some system options as context-sensitive config options;
2013-05-12, by wenzelm
load options for regular isabelle-process, not just for Isar loop (relevant for numerous low-level tools) -- NB: Isabelle_Process manages options via protocol message;
2013-05-12, by wenzelm
support for system options as context-sensitive config options;
2013-05-12, by wenzelm
tuned signature;
2013-05-12, by wenzelm
tuned comments;
2013-05-12, by wenzelm
support for options as preferences;
2013-05-12, by wenzelm
more operations in accordance to Scala version;
2013-05-12, by wenzelm
more systematic access to options default;
2013-05-12, by wenzelm
full default options for Isabelle_Process and Build;
2013-05-12, by wenzelm
decentralized historic settings;
2013-05-12, by wenzelm
removed obsolete test_markup;
2013-05-12, by wenzelm
Proof General interaction always uses Isar loop;
2013-05-12, by wenzelm
proper context;
2013-05-12, by wenzelm
merged
2013-05-11, by wenzelm
more direct PGIP/Emacs processing and output;
2013-05-11, by wenzelm
more direct interpretation of "askprefs" and "setpref", which appear to be the only PGIP command used in PG 3.7.1.1, 4.1, 4.2;
2013-05-11, by wenzelm
removed redundant modules;
2013-05-11, by wenzelm
removed some obsolete PGIP/PGEclipse material;
2013-05-11, by wenzelm
never open structure Unsynchronized (cf. "implementation" manual);
2013-05-11, by wenzelm
prefer explicitly qualified exceptions, which is particular important for robust handlers;
2013-05-11, by wenzelm
avoid PolyML.makestring, even in dead code;
2013-05-11, by wenzelm
fixed bug introduced when reintroducing set constructor, and visible when applying <= to 2- or more-ary relations, e.g. "(R::'a=>'a=>bool) <= R"
2013-05-11, by blanchet
don't apply an unnecessary morphism
2013-05-10, by kuncar
tuned
2013-05-10, by nipkow
relator coinduction for codatatypes
2013-05-09, by traytel
standard ivl notation [l,h]
2013-05-09, by nipkow
merged
2013-05-09, by nipkow
tuned
2013-05-08, by nipkow
avoid polymorphic uncurried aliases with more arguments than there are arguments in the most general type of a HOL constant, to dodge issues at declaration time
2013-05-08, by blanchet
proper unmangling -- the bug is visible when "uncurried_aliases" is enabled with Alt-Ergo or Poly. SPASS
2013-05-08, by blanchet
use right default for "uncurried_aliases" with polymorphic SPASS
2013-05-08, by blanchet
relator induction for datatypes
2013-05-08, by traytel
store proper theorems even for fixed points that have no passive live variables
2013-05-08, by traytel
stronger monotonicity property for relators
2013-05-08, by traytel
make tactic actually work for op = as relator
2013-05-08, by traytel
tuned
2013-05-08, by nipkow
hide Fin on output
2013-05-08, by nipkow
removed dead argument
2013-05-07, by blanchet
more robust iterator construction (needed for mutualized FPs)
2013-05-07, by blanchet
tuning
2013-05-07, by blanchet
removed dead internal constants/theorems
2013-05-07, by traytel
removed tracing
2013-05-07, by blanchet
export one more function
2013-05-07, by blanchet
added field to record
2013-05-07, by blanchet
tuning
2013-05-07, by blanchet
removed dead code
2013-05-07, by blanchet
move function to library
2013-05-07, by blanchet
tuning
2013-05-07, by blanchet
more
2013-05-07, by blanchet
tuning
2013-05-07, by blanchet
code tuning
2013-05-07, by blanchet
merge
2013-05-07, by blanchet
refactoring
2013-05-07, by blanchet
export one more function + tuning
2013-05-07, by blanchet
do not unfold the definition of the relator as it is not defined in terms of srel anymore
2013-05-07, by traytel
tuned
2013-05-07, by traytel
got rid of the set based relator---use (binary) predicate based relator instead
2013-05-07, by traytel
tuned names + extended ML signature
2013-05-07, by blanchet
merged
2013-05-07, by nipkow
tuned name: filter -> constrain (longer but more intuitive)
2013-05-07, by nipkow
tuning
2013-05-07, by blanchet
imported patch refactor_coiter_constr
2013-05-07, by blanchet
tuned
2013-05-07, by nipkow
started factoring out coiter construction
2013-05-06, by blanchet
rationalize ML signature
2013-05-06, by blanchet
factor out construction of iterator
2013-05-06, by blanchet
tuning
2013-05-06, by blanchet
improved defns and proofs
2013-05-06, by nipkow
undo 46d911ab9170 since it causes problems
2013-05-06, by smolkas
allow '-'s in tptp ids to avoid problems with remote_vampire
2013-05-06, by smolkas
added preplay tracing
2013-05-06, by smolkas
handle dummy atp terms
2013-05-06, by smolkas
avoid dummy annotations; terminate preplay/compression if metis fails; fixed bug
2013-05-06, by smolkas
added informative error messages
2013-05-06, by smolkas
tail recursive version of map, for code generation, optionally
2013-05-06, by nipkow
simplified proofs
2013-05-06, by nipkow
tuning
2013-05-03, by blanchet
pass certain readability-enhancing Vampire options only when an Isar proof is needed
2013-05-03, by blanchet
added lemma
2013-05-03, by nipkow
added lemma
2013-05-03, by nipkow
renamings
2013-05-02, by blanchet
code tuning
2013-05-02, by blanchet
signature tuning
2013-05-02, by blanchet
removed dead code
2013-05-02, by blanchet
tuned signature
2013-05-02, by blanchet
store (co)induction rules in data structure
2013-05-02, by blanchet
tuning names
2013-05-02, by blanchet
got rid of needless library function (find_minimum)
2013-05-02, by blanchet
one more lib function
2013-05-02, by blanchet
export one more function
2013-05-02, by blanchet
rationalized data structure
2013-05-02, by blanchet
added and moved library functions (used in primrec code)
2013-05-02, by blanchet
tuned names -- co_ and un_ with underscore are to be understood as (co) and (un)
2013-05-02, by blanchet
tuning
2013-05-02, by blanchet
more code rationalization
2013-05-02, by blanchet
more code rationalization
2013-05-02, by blanchet
more code rationalization
2013-05-02, by blanchet
refactoring
2013-05-02, by blanchet
tuned
2013-05-02, by nipkow
renamed a few FP-related files, to make it clear that these are not the sum of LFP + GFP but rather shared basic libraries
2013-05-01, by blanchet
tuned
2013-05-01, by nipkow
tuned
2013-05-01, by nipkow
tuning
2013-04-30, by blanchet
export more functions (useful for primrec_new)
2013-04-30, by blanchet
further enrich data structure
2013-04-30, by blanchet
more
2013-04-30, by blanchet
rationalized terminology (iterator = fold or rec, xxfoo = (co)foo or (un)foo)
2013-04-30, by blanchet
added fields to database
2013-04-30, by blanchet
tuned data structure
2013-04-30, by blanchet
renamed records
2013-04-30, by blanchet
added constructors to data structure
2013-04-30, by blanchet
added pre-BNFs to database
2013-04-30, by blanchet
lowercase type constructor, for consistency (cf. fp_result not FP_result nor FP_Result)
2013-04-30, by blanchet
renamed "bnf_def" keyword to "bnf" (since it's not a definition, but rather a registration)
2013-04-30, by blanchet
Added maps, sets, rels to "simps" thm collection
2013-04-30, by blanchet
tuned
2013-04-30, by nipkow
comment tuning
2013-04-30, by blanchet
tuning
2013-04-30, by blanchet
tuning
2013-04-30, by blanchet
tuning
2013-04-30, by blanchet
signature tuning
2013-04-30, by blanchet
whitespace tuning
2013-04-30, by blanchet
tuned signature
2013-04-30, by blanchet
canonical names of classes
2013-04-30, by nipkow
merged
2013-04-29, by blanchet
register all (co)datatypes in local data
2013-04-29, by blanchet
create data structure for storing (co)datatype information
2013-04-29, by blanchet
avoid empty isabelletags.sty for the sake of arXiv;
2013-04-29, by wenzelm
merged
2013-04-29, by wenzelm
cygwin_root as optional argument;
2013-04-29, by wenzelm
use record instead of big tuple
2013-04-29, by blanchet
clarified module dependencies: avoid Properties and Document introding minimal "PIDE";
2013-04-29, by wenzelm
merge
2013-04-29, by blanchet
use base names, not full names
2013-04-29, by blanchet
tune signatures
2013-04-29, by blanchet
tuning
2013-04-29, by blanchet
tuning
2013-04-29, by blanchet
removed unreferenced thm
2013-04-29, by blanchet
tuned function signatures
2013-04-29, by blanchet
factored out derivation of coinduction, unfold, corec
2013-04-29, by blanchet
code tuning
2013-04-29, by blanchet
factored out derivation of induction principles, folds and recs, in preparation for reduction of nested to mutual
2013-04-29, by blanchet
tuned
2013-04-29, by nipkow
tuned operator precedence
2013-04-29, by traytel
use record instead of huge tuple
2013-04-29, by blanchet
renamed BNF "(co)data" commands to names that are closer to their final names
2013-04-29, by blanchet
tuned
2013-04-29, by nipkow
tuned
2013-04-29, by nipkow
tuned
2013-04-29, by nipkow
tuned
2013-04-28, by nipkow
Clarified confusing sentence in locales tutorial.
2013-04-27, by ballarin
uniform Proof.context for hyp_subst_tac;
2013-04-27, by wenzelm
tuned ML and thy file names
2013-04-27, by blanchet
merged
2013-04-26, by blanchet
for compatibility, generate recursor arguments in the same order as old package
2013-04-26, by blanchet
tuning in preparation for actual changes
2013-04-26, by blanchet
started working on compatibility with old package's recursor
2013-04-26, by blanchet
simplified def
2013-04-26, by nipkow
more standard argument order
2013-04-26, by nipkow
more intuitive syntax for equality-style discriminators of nullary constructors
2013-04-26, by blanchet
updated keywords
2013-04-26, by blanchet
less
more
|
(0)
-30000
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
tip