Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-192
+192
+1000
+3000
+10000
+30000
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.
more user aliases;
2011-09-24, by wenzelm
fixed IsaMakefile action for HOL-TPTP.
2011-09-24, by sultana
prefer socket comminication on Cygwin, which is more stable here than fifos;
2011-09-23, by wenzelm
tuned proof;
2011-09-23, by wenzelm
made SML/NJ happy;
2011-09-23, by wenzelm
discontinued stream-based Socket_IO, which causes too many problems with Poly/ML and SML/NJ (reverting major parts of 5c0b0d67f9b1);
2011-09-23, by wenzelm
updated header;
2011-09-23, by wenzelm
merged;
2011-09-23, by wenzelm
reintroduced E-SInE now that it's unexpectedly working again (thanks to Geoff)
2011-09-23, by blanchet
first step towards extending Minipick with more translations
2011-09-23, by blanchet
Include keywords print_coercions and print_coercion_maps
2011-09-23, by berghofe
local coercion insertion algorithm to support complex coercions
2011-08-17, by traytel
printing and deleting of coercions
2011-08-17, by traytel
raw unbuffered socket IO, which bypasses the fragile BinIO layer in Poly/ML 5.4.x;
2011-09-23, by wenzelm
default print mode for Isabelle/Scala, not just Isabelle/jEdit;
2011-09-23, by wenzelm
augment existing print mode;
2011-09-23, by wenzelm
explicit option for socket vs. fifo communication;
2011-09-23, by wenzelm
tuned proof;
2011-09-23, by wenzelm
synchronized section names with manual
2011-09-23, by blanchet
merged;
2011-09-23, by wenzelm
discontinued legacy theorem names from RealDef.thy
2011-09-22, by huffman
merged
2011-09-22, by huffman
discontinued HOLCF legacy theorem names
2011-09-22, by huffman
take out remote E-SInE -- it's broken and Geoff says it might take quite a while before he gets to it, plus it's fairly obsolete in the meantime
2011-09-22, by blanchet
Moved extraction part of Higman's lemma to separate theory to allow reuse in
2011-09-22, by berghofe
Removed hcentering and vcentering options, since they are not supported
2011-09-22, by berghofe
merged
2011-09-22, by berghofe
Added documentation for HOL-SPARK
2011-09-22, by berghofe
drop partial monomorphic instances in Metis, like in Sledgehammer
2011-09-22, by blanchet
better type reconstruction -- prevents ill-instantiations in proof replay
2011-09-22, by blanchet
NEWS: mention replacement lemmas for the removed ones in Complete_Lattices
2011-09-22, by hoelzl
changing quickcheck_timeout to 30 seconds in mutabelle's testing
2011-09-22, by bulwahn
adding post-processing of terms to narrowing-based Quickcheck
2011-09-22, by bulwahn
HOL/ex/ROOT.ML: only list BinEx once
2011-09-21, by huffman
merged
2011-09-21, by huffman
remove redundant instantiation ereal :: power
2011-09-21, by huffman
reintroduced Minipick as Nitpick example
2011-09-21, by blanchet
tuned comment
2011-09-21, by blanchet
merged
2011-09-21, by huffman
Extended_Real_Limits: generalize some lemmas
2011-09-20, by huffman
add lemmas within_empty and tendsto_bot;
2011-09-20, by huffman
made SML/NJ happy;
2011-09-22, by wenzelm
abstract System_Channel in ML (cf. Scala version);
2011-09-22, by wenzelm
alternative Socket_Channel;
2011-09-21, by wenzelm
more abstract wrapping of fifos as System_Channel;
2011-09-21, by wenzelm
slightly more general Socket_IO as part of Pure;
2011-09-21, by wenzelm
more hints on Z3 configuration;
2011-09-21, by wenzelm
reduced default thread stack, to increase the success rate especially on Windows (NB: the actor worker farm tends to produce 100-200 threads for big sessions);
2011-09-21, by wenzelm
renamed inv -> filter
2011-09-21, by nipkow
Added proofs about narowing
2011-09-21, by nipkow
added missing makefile dependence
2011-09-21, by nipkow
added example
2011-09-21, by nipkow
tuned
2011-09-21, by nipkow
refined comment
2011-09-21, by nipkow
fixed two typos in IMP (by Jean Pichon)
2011-09-21, by kleing
merged
2011-09-21, by nipkow
Updated IMP to use new induction method
2011-09-20, by nipkow
New proof method "induction" that gives induction hypotheses the name IH.
2011-09-20, by nipkow
official status for UN_singleton
2011-09-20, by haftmann
tuned specification and lemma distribution among theories; tuned proofs
2011-09-20, by haftmann
more careful treatment of initial update, similar to output panel;
2011-09-20, by wenzelm
proper fact binding;
2011-09-20, by wenzelm
syntactic improvements and tuning names in the code generator due to Florian's code review
2011-09-20, by bulwahn
match types when applying mono_thm -- previous export generalizes type variables;
2011-09-20, by krauss
fixed headers;
2011-09-19, by wenzelm
less ambiguous syntax;
2011-09-19, by wenzelm
tuned proofs;
2011-09-19, by wenzelm
merged
2011-09-19, by wenzelm
catch PatternMatchFail exceptions in narrowing-based quickcheck
2011-09-19, by bulwahn
removing superfluous definition in the quickcheck narrowing invocation as the code generator now generates valid Haskell code with necessary type annotations without a separate definition
2011-09-19, by bulwahn
ensuring that some constants are generated in the source code by adding calls in ensure_testable
2011-09-19, by bulwahn
adding abstraction layer; more precise function names
2011-09-19, by bulwahn
adding type annotations more aggressively and redundantly to make code generation more reliable even when special printers for some constants are used
2011-09-19, by bulwahn
determining the fastype of a case-pattern but ignoring dummy type constructors that were added as markers for type annotations
2011-09-19, by bulwahn
only annotating constants with sort constraints
2011-09-19, by bulwahn
also adding type annotations for the dynamic invocation
2011-09-19, by bulwahn
removed legacy lemmas in Complete_Lattices
2011-09-19, by noschinl
increasing quickcheck timeout to reduce spurious test failures due to massive parallel invocations and bad scheduling
2011-09-19, by bulwahn
more isatest stats;
2011-09-19, by wenzelm
refined Symbol.is_symbolic -- cover recoded versions as well;
2011-09-19, by wenzelm
double clicks switch to document node buffer;
2011-09-19, by wenzelm
tuned;
2011-09-19, by wenzelm
explicit border independent of UI (cf. ad5883642a83, 2bec3b7514cf);
2011-09-19, by wenzelm
at least 2 worker threads to ensure some degree of lifeness, notably for asynchronous Document.print_state;
2011-09-19, by wenzelm
instantaneous cleanup (NB: VIEWER should be synchronous, cf. dd25b3055c4e);
2011-09-19, by wenzelm
unique file names via serial numbers, to allow files like "root" or multiple files with same base name;
2011-09-19, by wenzelm
imitate Apple in setting initial shell PATH -- especially relevant for MacTeX, MacPorts etc.;
2011-09-19, by wenzelm
merged
2011-09-18, by huffman
numeral_simprocs.ML: use HOL_basic_ss instead of HOL_ss for internal normalization proofs of cancel_factor simprocs, to avoid splitting if-then-else
2011-09-15, by huffman
removed obsolete patches for PG 4.1;
2011-09-18, by wenzelm
additional space for borderless UI;
2011-09-18, by wenzelm
more robust treatment of empty insets (NB: border may be null on some UIs, e.g. Windows);
2011-09-18, by wenzelm
explicit master_dir as part of header -- still required (for Cygwin) since Scala layer does not pass file content yet;
2011-09-18, by wenzelm
isatest settings for macbroy6 (Mac OS X Lion);
2011-09-18, by wenzelm
more Mac OS reference hardware;
2011-09-18, by wenzelm
updated to SML/NJ 110.73;
2011-09-18, by wenzelm
tentative announcement based on current NEWS;
2011-09-18, by wenzelm
tuned;
2011-09-18, by wenzelm
separated NEWS for Isabelle2011 from Isabelle2011-1 (cf. e1139e612b55);
2011-09-18, by wenzelm
updated for release;
2011-09-18, by wenzelm
tuned;
2011-09-18, by wenzelm
updated generated file;
2011-09-18, by wenzelm
updated Complete_Lattices;
2011-09-18, by wenzelm
some tuning and re-ordering for release;
2011-09-18, by wenzelm
misc tuning for release;
2011-09-18, by wenzelm
more contributors;
2011-09-18, by wenzelm
tuned proofs;
2011-09-18, by wenzelm
tweak keyboard shortcuts for Mac OS X;
2011-09-18, by wenzelm
explicit check_file wrt. jEdit VFS, to avoid slightly confusing empty buffer after IO error;
2011-09-18, by wenzelm
finite sequences as useful as introductory example;
2011-09-18, by wenzelm
discontinued hard-wired JAVA_HOME treatment for Mac OS X (cf. f471a2fb9a95), which can cause confusions of "isabelle java" vs. "isabelle scala" -- moved settings to external component;
2011-09-18, by wenzelm
graph traversal in topological order;
2011-09-18, by wenzelm
Document.Node.Name convenience;
2011-09-17, by wenzelm
more precise painting;
2011-09-17, by wenzelm
more elaborate Node_Renderer, which paints node_name.theory only;
2011-09-17, by wenzelm
raised default log level -- to avoid confusing warning about scala.tools.nsc.plugins.Plugin, which is mistaken as jEdit plugin;
2011-09-17, by wenzelm
tuned signature;
2011-09-17, by wenzelm
more careful traversal of theory dependencies to retain standard import order;
2011-09-17, by wenzelm
sane default for class Thy_Load;
2011-09-17, by wenzelm
removed obsolete patches for PG 4.1;
2011-09-17, by wenzelm
specific bundle for x86_64-linux, which is especially important for JRE due to its extra library dependencies;
2011-09-17, by wenzelm
added "isabelle scalac" convenience;
2011-09-17, by wenzelm
Symbol.explode as in ML;
2011-09-17, by wenzelm
ignore OUTPUT to avoid spam -- jEdit menu "Troubleshooting / Activity Log" should be sufficient;
2011-09-17, by wenzelm
dropped unused argument – avoids problem with SML/NJ
2011-09-17, by haftmann
tuned spacing
2011-09-17, by haftmann
tuned
2011-09-17, by haftmann
tuned post fixpoint setup
2011-09-17, by nipkow
merged
2011-09-17, by nipkow
when applying induction rules, remove names of assumptions that come
2011-09-16, by nipkow
remove stray "using [[simp_trace]]"
2011-09-16, by noschinl
tune indenting
2011-09-16, by noschinl
removed unused legacy lemma names, some comment cleanup.
2011-09-16, by kleing
removed word_neq_0_conv from simpset, it's almost never wanted.
2011-09-16, by kleing
removed further legacy rules from Complete_Lattices
2011-09-15, by hoelzl
NEWS on Complete_Lattices, Lattices
2011-09-15, by noschinl
tail recursive proof preprocessing (needed for huge proofs)
2011-09-15, by blanchet
tuning
2011-09-15, by blanchet
merged
2011-09-15, by nipkow
revised AbsInt and added widening and narrowing
2011-09-15, by nipkow
updated comment
2011-09-14, by haftmann
updated generated code
2011-09-14, by haftmann
tuned
2011-09-13, by haftmann
renamed Complete_Lattices lemmas, removed legacy names
2011-09-14, by hoelzl
merged
2011-09-14, by noschinl
create central list for language extensions used by the haskell code generator
2011-09-14, by noschinl
observe distinction between sets and predicates
2011-09-14, by boehmes
merged
2011-09-14, by nipkow
cleand up AbsInt fixpoint iteration; tuned syntax
2011-09-14, by nipkow
tuned proofs
2011-09-13, by huffman
tuned proofs
2011-09-13, by huffman
remove some redundant [simp] declarations;
2011-09-13, by huffman
tune proofs
2011-09-13, by noschinl
tune simpset for Complete_Lattices
2011-09-13, by noschinl
merged
2011-09-13, by bulwahn
added lemma motivated by a more specific lemma in the AFP-KBPs theories
2011-09-13, by bulwahn
simplified unsound proof detection by removing impossible case
2011-09-13, by blanchet
correcting NEWS
2011-09-13, by bulwahn
correcting theory name and dependencies
2011-09-13, by bulwahn
renamed AList_Impl to AList
2011-09-13, by bulwahn
fastsimp -> fastforce in doc
2011-09-13, by nipkow
fix typo
2011-09-12, by huffman
shorten proof of frontier_straddle
2011-09-12, by huffman
NEWS and CONTRIBUTORS
2011-09-12, by huffman
remove redundant lemma Lim_sequentially in favor of lemma LIMSEQ_def
2011-09-12, by huffman
simplify proofs using LIMSEQ lemmas
2011-09-12, by huffman
remove trivial lemma Lim_at_iff_LIM
2011-09-12, by huffman
fix typos
2011-09-12, by huffman
NEWS for euclidean_space class
2011-09-12, by huffman
move lemmas about complex number 'i' to Complex.thy and Library/Inner_Product.thy
2011-09-12, by huffman
adding NEWS and CONTRIBUTORS
2011-09-12, by hoelzl
merged
2011-09-12, by bulwahn
correcting imports after splitting and renaming AssocList
2011-09-12, by bulwahn
tuned
2011-09-12, by bulwahn
moving connection of association lists to Mappings into a separate theory
2011-09-12, by bulwahn
adding NEWS and CONTRIBUTORS
2011-09-12, by bulwahn
tuned some symbol that probably went there by some strange encoding issue
2011-09-12, by bulwahn
added my contributions to NEWS and CONTRIBUTORS
2011-09-12, by blanchet
fixed type intersection (again)
2011-09-12, by blanchet
consistent option naming
2011-09-12, by blanchet
NEWS fastsimp -> fastforce
2011-09-12, by nipkow
new fastforce replacing fastsimp - less confusing name
2011-09-12, by nipkow
merged
2011-09-11, by wenzelm
NEWS for Library/Product_Lattice.thy
2011-09-11, by huffman
misc tuning and clarification;
2011-09-11, by wenzelm
merged
2011-09-11, by wenzelm
merged
2011-09-11, by huffman
tuned proofs
2011-09-11, by huffman
Library/Saturated.thy: 'Sat' abbreviates 'of_nat'
2011-09-11, by huffman
more CONTRIBUTORS;
2011-09-11, by wenzelm
persistent ISABELLE_INTERFACE_CHOICE;
2011-09-11, by wenzelm
explicit choice of interface;
2011-09-11, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-192
+192
+1000
+3000
+10000
+30000
tip