Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+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.
only conceal primitive definition theorems, not predicate names
2010-09-09, by haftmann
merged
2010-09-08, by haftmann
modernized primrec
2010-09-08, by haftmann
Markup_Tree is already scalable;
2010-09-10, by wenzelm
Isabelle_Markup.tooltip: explicit indication of ML;
2010-09-10, by wenzelm
Future.promise: more robust treatment of concurrent abort vs. fulfill (amending 047c96f41455);
2010-09-10, by wenzelm
primitive use_text: let interrupts pass unhindered;
2010-09-10, by wenzelm
Isabelle.load_icon with some sanity checks;
2010-09-09, by wenzelm
ML_Compiler.eval: reported positions need to contain offset, to avoid displaced reports due to synthesized line numbers;
2010-09-09, by wenzelm
NEWS: some notes on interrupts;
2010-09-09, by wenzelm
refined Runtime.toplevel_error/Document.run_command: let interrupts pass unhindered;
2010-09-09, by wenzelm
removed dead code;
2010-09-09, by wenzelm
avoid handling interrupts in user code;
2010-09-09, by wenzelm
Meson.make_clauses_unsorted: removed spurious debug code stemming from 5146d640aa4a -- must not handle arbitrary exceptions in user space;
2010-09-09, by wenzelm
main command loops are supposed to be uninterruptible -- no special treatment here;
2010-09-09, by wenzelm
Exn.is_interrupt: include interrupts that have passed through the IO layer;
2010-09-09, by wenzelm
more abstract treatment of interrupts in structure Exn -- hardly ever need to mention Interrupt literally;
2010-09-09, by wenzelm
avoid mixing of static and runtime errors in compiler output, to accomodate Proof General;
2010-09-09, by wenzelm
ML_Compiler.eval: discontinued extra "Static Errors" of raw Poly/ML;
2010-09-08, by wenzelm
isabelle-jedit.css: suppress "location" markup, which indicates extra positional information intended for plain-old TTY mode;
2010-09-08, by wenzelm
ML_Compiler.eval: more careful printing of messages and regular output, trying to accomodate Poly/ML, Proof General, Isabelle/Scala/jEdit at the same time;
2010-09-08, by wenzelm
clarified -- inlined ML_Env.local_context;
2010-09-08, by wenzelm
merged
2010-09-08, by wenzelm
restricting invocation only if PROLOG_HOME is set
2010-09-08, by bulwahn
tuned proofs (based on fancy gutter icons in Isabelle/jEdit);
2010-09-08, by wenzelm
merge
2010-09-08, by blanchet
remove "safe" (as suggested by Tobias) and added "arith" to "try"
2010-09-08, by blanchet
remove "minipick" (the toy version of Nitpick) and some tests;
2010-09-06, by blanchet
use Future.fork rather than Thread.fork, so that the thread is part of the global thread management
2010-09-06, by blanchet
fix editor
2010-09-06, by blanchet
merged
2010-09-08, by wenzelm
merged
2010-09-08, by paulson
tidied using inductive_simps
2010-09-08, by paulson
NEWS
2010-09-08, by haftmann
removed ancient constdefs command
2010-09-08, by haftmann
put expand_(fun/set)_eq back in as synonyms, for compatibility
2010-09-08, by nipkow
set up Nil and Cons to work as fixrec patterns
2010-09-07, by huffman
merged
2010-09-07, by haftmann
updated generated document
2010-09-07, by haftmann
only write ghc pragma when writing to a file
2010-09-07, by haftmann
added flat_program; tuned signature
2010-09-07, by haftmann
dropped ancient deresolve_base; plain_const_syntax also needs modification of instance statement
2010-09-07, by haftmann
moved flat_program to code_namespace
2010-09-07, by haftmann
dropped outdated substitution
2010-09-07, by haftmann
Haskell uses generic flat_program combinator
2010-09-07, by haftmann
factored out build_module_namespace
2010-09-07, by haftmann
added generic flat_program procedure
2010-09-07, by haftmann
using the proposed modes for starting the fixpoint iteration in the mode analysis
2010-09-07, by bulwahn
merged
2010-09-07, by nipkow
renamed expand_*_eq in HOLCF as well
2010-09-07, by nipkow
expand_fun_eq -> ext_iff
2010-09-07, by nipkow
merged
2010-09-07, by bulwahn
lower expectation in Reg exp example
2010-09-07, by bulwahn
renewing specification in example file; adding invocation in example file
2010-09-07, by bulwahn
handling collection of simprules as sets rather than as lists
2010-09-07, by bulwahn
stating errors in error messages more verbose in predicate compiler
2010-09-07, by bulwahn
raising an exception instead of guessing some reasonable behaviour for this function
2010-09-07, by bulwahn
using linear find_least instead of sorting in the mode analysis of the predicate compiler
2010-09-07, by bulwahn
adding code attribute to definition of equality of finite sets for executability of equality of finite sets
2010-09-07, by bulwahn
adapting example files
2010-09-07, by bulwahn
adding the Reg_Exp example
2010-09-07, by bulwahn
towards time limiting the prolog execution
2010-09-07, by bulwahn
adding IMP quickcheck examples
2010-09-07, by bulwahn
adding the CFG example to the build process
2010-09-07, by bulwahn
adding a List example (challenge from Tobias) for counterexample search
2010-09-07, by bulwahn
adding dependencies to IsaMakefile; increasing negative search limit for predicate_compile_quickcheck; adding tracing of introduction rules in code_prolog
2010-09-07, by bulwahn
disposed some old TODO/FIXME;
2010-09-08, by wenzelm
Document_View: select gutter message icons from markup over line range, not full range results;
2010-09-07, by wenzelm
tuned properties;
2010-09-07, by wenzelm
moved token markup tables to isabelle_markup.scala;
2010-09-07, by wenzelm
concentrate Isabelle specific physical rendering markup selection in isabelle_markup.scala;
2010-09-07, by wenzelm
simplified Markup_Tree.select: Stream instead of Iterator (again), explicit Option instead of default;
2010-09-07, by wenzelm
Document_View: more precise painting of gutter icons, only if line selection area is sufficiently large;
2010-09-07, by wenzelm
basic support for warning/error gutter icons;
2010-09-07, by wenzelm
Document_View: some markup for main inner syntax categories;
2010-09-07, by wenzelm
Command.State.accumulate: check actual source range;
2010-09-07, by wenzelm
Isar_Document.reported_positions: slightly more robust treatment of positions outside the command range, notably parsing beyond EOF;
2010-09-07, by wenzelm
highlight bad range of nested error (here from inner parsing);
2010-09-07, by wenzelm
Isar_Document.reported_positions: exclude proof state output;
2010-09-07, by wenzelm
Document_View: less aggressive background coloring, departing from classic PG highlighting;
2010-09-07, by wenzelm
report token range after inner parse error -- often provides important clues about misunderstanding concerning lexical phase;
2010-09-07, by wenzelm
slightly more robust Plugin.stop -- components might refer to Isabelle.system even after shutdown;
2010-09-07, by wenzelm
turned show_hyps and show_tags into proper configuration option;
2010-09-06, by wenzelm
discontinued obsolete ProofContext.prems_limit;
2010-09-06, by wenzelm
ML_Context.thm and ML_Context.thms no longer pervasive;
2010-09-06, by wenzelm
more explicit indication of Config.raw options, which are only needed for bootstrapping Pure;
2010-09-06, by wenzelm
merged
2010-09-06, by wenzelm
When comparing Floats use integers instead of reals (represented as rationals), generates less code when Floats are used.
2010-09-06, by hoelzl
isatest: back to polyml-5.3.0 due to unresolved stability issues of polyml-5.4.0 and HOL/Decision_Procs/Approximation_Ex.thy;
2010-09-06, by wenzelm
more antiquotations;
2010-09-06, by wenzelm
ML_Context.thm;
2010-09-06, by wenzelm
more explicit HOL-Proofs sessions, including former ex/Hilbert_Classical.thy which works in parallel mode without the antiquotation option "margin" (which is still critical);
2010-09-06, by wenzelm
modernized session ROOT setup;
2010-09-06, by wenzelm
some results of concurrency code inspection;
2010-09-06, by wenzelm
merged;
2010-09-06, by wenzelm
mention ~/.isabelle/etc/settings file
2010-09-06, by blanchet
make remote ATP invocation work for those people who need to go through a proxy;
2010-09-06, by blanchet
enabled do notation for option type
2010-09-05, by krauss
removed duplicate lemma
2010-09-05, by krauss
added Option.bind
2010-09-05, by krauss
merged
2010-09-04, by haftmann
printing combinator for hierarchical programs
2010-09-04, by haftmann
merged
2010-09-04, by haftmann
add lemma cont2cont_Let_simple
2010-09-04, by huffman
add lemma cont2cont_split_simple
2010-09-04, by huffman
add List_Cpo.thy to HOLCF/Library
2010-09-04, by huffman
dropped names from serializer interface
2010-09-04, by haftmann
added more explicit warning
2010-09-04, by haftmann
ML_Context.ml_store_thm(s): operate on thread context instead of Unsynchronized.ref;
2010-09-06, by wenzelm
use setmp_noncritical for PGIP, which is presumably sequential (PG clone);
2010-09-05, by wenzelm
use setmp_noncritical for sequential Pure bootstrap;
2010-09-05, by wenzelm
turned show_brackets into proper configuration option;
2010-09-05, by wenzelm
Syntax.standard_parse_term: eliminated redundant Pretty.pp;
2010-09-05, by wenzelm
structure Syntax: define "interfaces" before actual implementations;
2010-09-05, by wenzelm
turned show_sorts/show_types into proper configuration options;
2010-09-05, by wenzelm
pretty printing: prefer regular Proof.context over Pretty.pp, which is mostly for special bootstrap purposes involving theory merge, for example;
2010-09-05, by wenzelm
refined treatment of multi-line subexpressions;
2010-09-04, by wenzelm
basic support for subexpression highlighting (see also gatchan.jedit.hyperlinks.HyperlinkManager/HyperlinkTextAreaPainter);
2010-09-04, by wenzelm
updated configuration options;
2010-09-04, by wenzelm
recovered options for goal antiquotations from f45d332a90e3: actually pass context to Proof.pretty_goals (see also 45facd8f358e);
2010-09-04, by wenzelm
turned eta_contract into proper configuration option;
2010-09-03, by wenzelm
turned show_structs into proper configuration option;
2010-09-03, by wenzelm
configuration options Syntax.ambiguity_enabled (inverse of former Syntax.ambiguity_is_error), Syntax.ambiguity_level (with Isar attribute "syntax_ambiguity_level"), Syntax.ambiguity_limit;
2010-09-03, by wenzelm
pretty_goals: turned some global references and function arguments into configuration options (goals_limit = 10, goals_total = true, show_main_goal = false) depending on the context;
2010-09-03, by wenzelm
tuned comment;
2010-09-03, by wenzelm
merged
2010-09-03, by wenzelm
merged
2010-09-03, by haftmann
QND_FLAG is a shell variable, not a string
2010-09-03, by haftmann
modernized session ROOT;
2010-09-03, by wenzelm
disposed left-over user preferences;
2010-09-03, by wenzelm
turned show_all_types into proper configuration option;
2010-09-03, by wenzelm
treat show_free_types as plain ML option, without the extras of global default and registration in the attribute name space -- NB: 'print_configs' only shows the latter;
2010-09-03, by wenzelm
more explicit Config.declare vs. Config.declare_global;
2010-09-03, by wenzelm
turned show_no_free_types into proper configuration option show_free_types, with flipped polarity;
2010-09-03, by wenzelm
remove code I submitted accidentally
2010-09-03, by blanchet
merged
2010-09-03, by blanchet
disable "definitional CNF";
2010-09-03, by blanchet
redisable Nitpick from Cygwin, until I've investigated the issue
2010-09-03, by blanchet
show the number of facts for each prover in "verbose" mode
2010-09-02, by blanchet
fix bug in "debug" mode
2010-09-02, by blanchet
make sure "Unknown ATP" errors reach the users -- i.e. don't generate them from a thread
2010-09-02, by blanchet
If Geoff puts some important message in his TPTP problems (e.g., money requests), we should show them to the user
2010-09-02, by blanchet
fix trivial "x = x" fact detection
2010-09-02, by blanchet
merged
2010-09-03, by wenzelm
merged
2010-09-03, by haftmann
merged
2010-09-02, by haftmann
hand out deresolver from serializer invocation
2010-09-02, by haftmann
Revert bij_betw changes to simp set (Problem in afp/Ordinals_and_Cardinals)
2010-09-02, by hoelzl
merged
2010-09-02, by hoelzl
Updated proofs in Dining Cryptographers theory
2010-09-02, by hoelzl
Corrected definition and hence removed sorry.
2010-09-02, by hoelzl
Moved lemmas to appropriate locations
2010-09-02, by hoelzl
merged
2010-09-02, by hoelzl
merged
2010-09-02, by hellerar
measure unique
2010-09-02, by hellerar
merge
2010-09-01, by hellerar
move lemmas to correct theory files
2010-09-02, by hoelzl
factorizable measurable functions
2010-08-27, by hoelzl
Introduced sigma algebra generated by function preimages.
2010-08-27, by hoelzl
vimage of measurable function is a measure space
2010-08-27, by hoelzl
Measurable on product space is equiv. to measurable components
2010-08-27, by hoelzl
Measurable on euclidean space is equiv. to measurable components
2010-08-27, by hoelzl
preimages of open sets over continuous function are open
2010-08-27, by hoelzl
added definition of conditional expectation
2010-08-27, by hoelzl
proved existence of conditional expectation
2010-08-27, by hoelzl
introduced integration on subalgebras
2010-08-26, by hoelzl
changed definition of dynkin; replaces proofs by metis calles
2010-08-26, by hoelzl
dynkin
2010-08-26, by hellerar
dynkin system
2010-08-26, by hellerar
merged
2010-09-02, by hoelzl
Fixes lemma names
2010-09-02, by hoelzl
NEWS
2010-09-02, by hoelzl
Introduce surj_on and replace surj and bij by abbreviations.
2010-09-02, by hoelzl
Permutation implies bij function
2010-09-02, by hoelzl
bij <--> bij_betw
2010-09-02, by hoelzl
Add filter_remove1
2010-09-02, by hoelzl
Add lessThan_Suc_eq_insert_0
2010-09-02, by hoelzl
merged
2010-09-02, by haftmann
updated
2010-09-02, by haftmann
set printmode while marking
2010-09-02, by haftmann
updated
2010-09-02, by haftmann
avoid reference to theory Ferrack altogether
2010-09-02, by haftmann
more canonical theory setup
2010-09-02, by haftmann
set depth to 1
2010-09-02, by haftmann
avoid theory Imperative_HOL altogether
2010-09-02, by haftmann
adapted to change eq -> equal
2010-09-02, by haftmann
corrected printmode handling
2010-09-02, by haftmann
swapped slip
2010-09-02, by haftmann
updated
2010-09-02, by haftmann
restored and added surpression of case combinators
2010-09-02, by haftmann
dropped superfluous presentation names
2010-09-02, by haftmann
manage statement selection for presentation wholly through markup
2010-09-02, by haftmann
formal markup of generated code for statements
2010-09-02, by haftmann
removed namespace stuff from code_printer
2010-09-02, by haftmann
merged
2010-09-02, by blanchet
reenable Nitpick on Cygwin;
2010-09-02, by blanchet
merged;
2010-09-03, by wenzelm
Proof.pretty_state: print everything in the foreground context to give users a chance to configure options, e.g. via "using [[show_consts]]";
2010-09-03, by wenzelm
turned show_consts into proper configuration option;
2010-09-03, by wenzelm
prefer regular Proof.context over background theory;
2010-09-03, by wenzelm
just one refute.ML;
2010-09-02, by wenzelm
use existing Integer.pow, despite its slightly odd argument order;
2010-09-02, by wenzelm
tuned whitespace and indentation, emphasizing the logical structure of this long text;
2010-09-02, by wenzelm
inner parsing: refrain from too many nested position reports to achieve more precise error feedback in the source;
2010-09-02, by wenzelm
Document_View: squiggly underline for messages;
2010-09-02, by wenzelm
added gfx_range convenience;
2010-09-02, by wenzelm
Isar_Document.reported_positions: more precise include/exclude, include root as last resort only;
2010-09-02, by wenzelm
Position.Range: exclude singularity (again);
2010-09-02, by wenzelm
merged
2010-09-02, by wenzelm
merged
2010-09-02, by blanchet
FIXME -> TODO (nothing is broken)
2010-09-02, by blanchet
Let MESON take an additional "preskolemization tactic", which can be used to put the goal in definitional CNF
2010-09-02, by blanchet
use definitional CNFs in Metis rather than plain CNF, following a suggestion by Joe Hurd;
2010-09-02, by blanchet
make definitional CNF translation code more robust in the presence of existential quantifiers in the "literals"
2010-09-02, by blanchet
formal framework for presentation of selected statements
2010-09-02, by haftmann
merged
2010-09-02, by haftmann
Table.map replaces Table.map'
2010-09-02, by haftmann
dropped dead code; tuned
2010-09-02, by haftmann
include names need not be considered as reserved any longer
2010-09-02, by haftmann
skip empty name bunches; fill up trailing positions with NONEs
2010-09-02, by haftmann
use code_namespace module for SML and OCaml code
2010-09-02, by haftmann
Table.map replaces Table.map'
2010-09-02, by haftmann
avoid cyclic modules
2010-09-02, by haftmann
merged
2010-09-02, by haftmann
simultaneous modification of statements: statement names
2010-09-01, by haftmann
simultaneous modification of statements
2010-09-01, by haftmann
explicit modify_stmt parameter
2010-09-01, by haftmann
Graph.map, in analogy to Table.map
2010-09-01, by haftmann
replaced Table.map' by Table.map
2010-09-01, by haftmann
merged
2010-09-01, by haftmann
tuned
2010-09-01, by haftmann
generalized hierarchical data structure over statements
2010-09-01, by haftmann
merged
2010-09-02, by haftmann
normalization is allowed to solve True
2010-09-02, by haftmann
merged
2010-09-02, by blanchet
merged
2010-09-02, by blanchet
cosmetics
2010-09-02, by blanchet
SNARK doesn't like facts
2010-09-02, by blanchet
show real CPU time
2010-09-02, by blanchet
factor out code shared by all ATPs so that it's run only once
2010-09-01, by blanchet
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip