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
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.
tuned tactic
2014-02-20, by traytel
tuned
2014-02-20, by haftmann
less flex-flex pairs
2014-02-20, by noschinl
less flex-flex pairs (thanks to Lars' statistics)
2014-02-20, by traytel
made tactics more robust
2014-02-20, by traytel
offical tool
2014-02-19, by haftmann
more convenient syntax for permanent interpretation
2014-02-19, by haftmann
aggiornamento for "interpretation with definitions": operate uniformly on theory and locale level under the brand of "permanent interpretation"
2014-02-19, by haftmann
move stronger rules into exercise
2014-02-20, by kleing
added a function that carries out all the reconstruction steps, for improved usability;
2014-02-19, by sultana
reconstruction framework for LEO-II's TPTP proofs;
2014-02-19, by sultana
made list of test files a parameter to timed_test in TPTP_Test.thy, and updated dependent definitions;
2014-02-19, by sultana
cleaned code used to produce a proof-graph;
2014-02-19, by sultana
improved configurability of DOT exporter;
2014-02-19, by sultana
behaviour of tptp_graph now depends on an envir variable to indicate whether to produce proof graph containing formulas or not;
2014-02-19, by sultana
experimented with presentation of DOT+LaTeX;
2014-02-19, by sultana
edges are now being shown in the proof graph;
2014-02-19, by sultana
added case for handling 'assumption' lines in Satallax proofs;
2014-02-19, by sultana
improved latex output: spacing between terms, and encoding terms in mathrm;
2014-02-19, by sultana
experimenting with improving DOT output, and embedding LaTeX code for formulas (rather than only giving the clause number);
2014-02-19, by sultana
added more node shapes (matched with roles);
2014-02-19, by sultana
updated NEWS
2014-02-19, by blanchet
merged 'List.set' with BNF-generated 'set'
2014-02-19, by blanchet
moved advanced folding into separate exercise
2014-02-19, by kleing
tuned definition
2014-02-19, by kleing
another simplification of internal codatatype construction
2014-02-19, by traytel
reflect 207538943038 in NEWS
2014-02-19, by traytel
reverted ba7392b52a7c: List_Prefix not needed anymore by codatatypes
2014-02-19, by traytel
removed not anymore used constants and theorems
2014-02-19, by traytel
simplifications of internal codatatype construction
2014-02-19, by traytel
adapted Nitpick to 'primrec' refactoring
2014-02-19, by blanchet
moved 'primrec' up (for real this time) and removed temporary 'old_primrec'
2014-02-19, by blanchet
rewrote a small portion of code to avoid dependency on low-level constant
2014-02-19, by blanchet
tuning
2014-02-19, by blanchet
provide more automation for type definitions (makes book exercises easier)
2014-02-19, by kleing
prepare two-stage 'primrec' setup
2014-02-18, by blanchet
tuning
2014-02-18, by blanchet
removed deadcode
2014-02-18, by blanchet
merged
2014-02-18, by blanchet
tuning
2014-02-18, by blanchet
made SML/NJ happier
2014-02-18, by blanchet
simplify proofs because of the stronger reflexivity prover
2014-02-18, by kuncar
delete or move now not necessary reflexivity rules due to 1726f46d2aa8
2014-02-18, by kuncar
implement the reflexivity prover as a monotonicity prover that proves R >= op=; derive "reflexivity" rules for relators from mono rules and eq rules
2014-02-18, by kuncar
merged
2014-02-18, by wenzelm
more markup;
2014-02-18, by wenzelm
proper term equality;
2014-02-18, by wenzelm
tuned message;
2014-02-18, by wenzelm
more uniform treatment of dockables and their standard actions;
2014-02-18, by wenzelm
standardized action and panel names;
2014-02-18, by wenzelm
tuned imports;
2014-02-18, by wenzelm
prefer concrete list append;
2014-02-18, by wenzelm
tuned whitespace;
2014-02-18, by wenzelm
more standard names for protocol and markup elements;
2014-02-18, by wenzelm
tuned whitespace;
2014-02-18, by wenzelm
tuned signature;
2014-02-18, by wenzelm
generic markup for embedded languages;
2014-02-18, by wenzelm
clarified special eol treatment (amending 3d55ef732cd7): allow last line to be empty, which means stop == end for second-last line;
2014-02-18, by wenzelm
more uniform/robust restriction of reported positions, e.g. relevant for "bad" markup due to unclosed comment in ML file;
2014-02-18, by wenzelm
subtle change of semantics of Thm.eq_thm, e.g. relevant for merge of src/HOL/Tools/Predicate_Compile/core_data.ML (cf. HOL-IMP);
2014-02-17, by wenzelm
always show PIDE positions as \<here> (0x002302 "House" from DejaVuSansMono);
2014-02-17, by wenzelm
hyperlink for visible positions;
2014-02-17, by wenzelm
more informative error;
2014-02-17, by wenzelm
more informative error;
2014-02-17, by wenzelm
removed not anymore used theorems
2014-02-18, by traytel
syntactic simplifications of internal (co)datatype constructions
2014-02-18, by traytel
follow up of 0819931d652d -- put right induction rule in the old data structure, repairs 'HOL-Proof'-based sessions
2014-02-18, by blanchet
simplified data structure by reducing the incidence of clumsy indices
2014-02-17, by blanchet
tuning
2014-02-17, by blanchet
made SML/NJ happy;
2014-02-17, by wenzelm
NEWS;
2014-02-17, by wenzelm
name derivations in 'primrec' for code extraction from proof terms
2014-02-17, by blanchet
renamed old 'primrec' to 'old_primrec' (until the new 'primrec' can be moved above 'Nat' in the theory dependencies)
2014-02-17, by blanchet
updated NEWS
2014-02-17, by blanchet
updated keywords
2014-02-17, by blanchet
renamed 'datatype_new_compat' to 'datatype_compat'
2014-02-17, by blanchet
renamed 'primrec_new' to 'primrec', overriding the old command (which it still uses as a fallback for old-style datatypes)
2014-02-17, by blanchet
tuning: moved code where it belongs
2014-02-17, by blanchet
have 'primrec_new' fall back on old 'primrec' when given old-style datatypes
2014-02-17, by blanchet
tuning
2014-02-17, by blanchet
more markup;
2014-02-17, by wenzelm
folded 'rel_option' into 'option_rel'
2014-02-16, by blanchet
folded 'list_all2' with the relator generated by 'datatype_new'
2014-02-16, by blanchet
removed final periods in messages for proof methods
2014-02-16, by blanchet
tuned proofs;
2014-02-16, by wenzelm
added a version of the Metis tactic that returns the unused facts
2014-02-16, by blanchet
tuned code
2014-02-16, by blanchet
more NEWS
2014-02-16, by blanchet
folded 'Option.set' into BNF-generated 'set_option'
2014-02-16, by blanchet
merged
2014-02-16, by wenzelm
prefer user-space tool within Pure.thy;
2014-02-16, by wenzelm
more markup;
2014-02-16, by wenzelm
more uniform rendering of text that is formally interpreted: avoid clash with inner markup;
2014-02-16, by wenzelm
recovered Isabelle_Sidekick_Markup from 9c53198dbb1c: snapshot requires Swing_Thread;
2014-02-16, by wenzelm
support ML antiquotations in Scala;
2014-02-16, by wenzelm
antiquotations within plain text: Scala version in accordance to ML;
2014-02-16, by wenzelm
tuned signature -- emphasize line-oriented aspect;
2014-02-16, by wenzelm
eliminated odd dislocation of keyword declaration and implementation (leftover from 318cd8ac1817)
2014-02-16, by haftmann
tuned whitespace;
2014-02-15, by wenzelm
removed odd comments -- inferred types are shown by Prover IDE;
2014-02-15, by wenzelm
removed dead code;
2014-02-15, by wenzelm
more uniform ML keyword markup;
2014-02-15, by wenzelm
merged
2014-02-15, by wenzelm
tuned;
2014-02-15, by wenzelm
clarified Isabelle/ML strings;
2014-02-15, by wenzelm
refined ML keyword styles;
2014-02-15, by wenzelm
isabelle-ml mode with separate token marker;
2014-02-15, by wenzelm
partial scans via ML_Lex.tokenize_context;
2014-02-15, by wenzelm
proper signature;
2014-02-14, by wenzelm
lexical syntax for SML (in Scala);
2014-02-14, by wenzelm
tuned;
2014-02-14, by wenzelm
removed dead code;
2014-02-14, by wenzelm
tuned signature (in accordance to ML version);
2014-02-14, by wenzelm
tuned proofs;
2014-02-14, by wenzelm
tuned signature -- separate Lexicon from Parsers (in accordance to ML version);
2014-02-14, by wenzelm
prefer latest ProofGeneral-4.2-1 by default;
2014-02-14, by wenzelm
updated thy_info.dependencies;
2014-02-14, by wenzelm
tuned message;
2014-02-14, by wenzelm
more integrity checks of theory names vs. full node names;
2014-02-14, by wenzelm
abstract type must be a type constructor; check it
2014-02-15, by kuncar
generate proper 'DtRec' indices in 'datatype_new_compat' for the case where some types are duplicated
2014-02-14, by blanchet
better handling of recursion through functions
2014-02-14, by blanchet
added examples/tests
2014-02-14, by blanchet
tuned code to allow mutualized corecursion through different functions with the same target type
2014-02-14, by blanchet
removed assumption in 'primrec_new' that a given constructor can only occur once
2014-02-14, by blanchet
generate unique names
2014-02-14, by blanchet
allow different functions to recurse on the same type, like in the old package
2014-02-14, by blanchet
improved 'datatype_new_compat': generate more fixpoint equations for types like 'datatype_new x = C (x list) (x list)' (here, one equation for each x list instead of a single for both), for higher compatibility + code generation attributes on the recursor
2014-02-14, by blanchet
made N2M more robust w.r.t. identical nested types
2014-02-14, by traytel
register bnfs for (co)datatypes under their proper name (lost in af71b753c459)
2014-02-14, by traytel
updated keywords;
2014-02-14, by wenzelm
restored old 'remotify' logic -- too many bugs were introduced when refactoring the code
2014-02-14, by blanchet
more (co)datatype docs
2014-02-14, by blanchet
hide 'rel' name -- this one is waiting to be merged with 'list_all2'
2014-02-14, by blanchet
updated docs to reflect the new 'free_constructors' syntax
2014-02-14, by blanchet
more precise spec rules for selectors
2014-02-14, by blanchet
removed needless robustness (no longer needed thanks to new syntax)
2014-02-14, by blanchet
aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax
2014-02-14, by blanchet
renamed 'wrap_free_constructors' to 'free_constructors' (cf. 'functor', 'bnf', etc.)
2014-02-14, by blanchet
renamed 'enriched_type' to more informative 'functor' (following the renaming of enriched type constructors to bounded natural functors)
2014-02-14, by blanchet
merged 'Option.map' and 'Option.map_option'
2014-02-14, by blanchet
merged 'List.map' and 'List.list.map'
2014-02-14, by blanchet
have 'Ctr_Sugar' register its 'Spec_Rules'
2014-02-14, by blanchet
register 'Spec_Rules' for new-style (co)datatypes
2014-02-14, by blanchet
added 'Spec_Rules' for 'primcorec'
2014-02-14, by blanchet
more integrity checks of theory names vs. full node names -- at least for the scope of a single use_thys (or "theories" section in ROOT);
2014-02-13, by wenzelm
added a bit of documentation for the different commands
2014-02-13, by blanchet
cleaner, complete proof in documentation, contributed by Dmitriy T.
2014-02-13, by blanchet
do the right thing with provers that exist only remotely (e.g. e_sine)
2014-02-13, by blanchet
more precise descripiton
2014-02-13, by kuncar
all_args_conv works also for zero arguments
2014-02-13, by kuncar
don't catch QOUT_THM_INTERNAL from the recursive call of parametrize_relation_conv
2014-02-13, by kuncar
Lifting: support a type variable as a raw type
2014-02-12, by kuncar
repaired logic for default provers -- ensures Z3 is kept if installed and configured as noncommercial
2014-02-13, by blanchet
avoid changing the state's context -- this results in transfer problems later with SMT, and hence preplay tactic failures
2014-02-13, by blanchet
removed hint that is seldom useful in practice
2014-02-13, by blanchet
reactivate some examples that still appear to work;
2014-02-13, by wenzelm
removed dead code;
2014-02-13, by wenzelm
explicit indication that redefining outer syntax commands is not supposed to happen -- NB: interactive mode requires global change of syntax;
2014-02-13, by wenzelm
do not redefine outer syntax commands;
2014-02-13, by wenzelm
tuned whitespace;
2014-02-13, by wenzelm
static repair of ML file -- untested (!) by default since 76965c356d2a;
2014-02-13, by wenzelm
iteration n in the 'default' vs. 'update_new' vs. 'update' saga -- 'update' makes sense now that we honor the canonical order on 'merge' (as opposed to raising 'DUP')
2014-02-12, by blanchet
don't hide constant forever, since it may appear in some 'primcorec'-generated theorems
2014-02-12, by blanchet
tuning
2014-02-12, by blanchet
HOL-IMP fastness
2014-02-12, by traytel
merged, resolving some conflicts;
2014-02-12, by wenzelm
eliminated hard tabs (assuming tab-width=2);
2014-02-12, by wenzelm
more platform notes;
2014-02-12, by wenzelm
tuned whitespace;
2014-02-12, by wenzelm
removed odd comments -- inferred types are shown by Prover IDE;
2014-02-12, by wenzelm
maintain blob edits within history, which is important for Snapshot.convert/revert;
2014-02-12, by wenzelm
more accurate eq_content;
2014-02-12, by wenzelm
clarified message_positions: cover alt_id as well;
2014-02-12, by wenzelm
maintain multiple command chunks and markup trees: for main chunk and loaded files;
2014-02-11, by wenzelm
common Command.Chunk for command source and auxiliary files (static Symbol.Index without actual String content);
2014-02-11, by wenzelm
tuned signature;
2014-02-11, by wenzelm
report (but ignore) markup within auxiliary files;
2014-02-11, by wenzelm
merged
2014-02-12, by Andreas Lochbihler
make integer_of_char and char_of_integer work with NBE and code_simp
2014-02-12, by Andreas Lochbihler
make lifting setup for String.literal local to prevent transfer from replacing STR ''...'' literals
2014-02-12, by Andreas Lochbihler
[mq]: news
2014-02-12, by blanchet
remove hidden fact about hidden constant from code generator setup
2014-02-12, by blanchet
for extraction -- use the exhaust rule that's registered with 'datatype_realizer.ML'
2014-02-12, by blanchet
compile
2014-02-12, by blanchet
updated certificates
2014-02-12, by blanchet
tuned message
2014-02-12, by blanchet
tabled, v.: postpone consideration of
2014-02-12, by blanchet
adapted to renaming of 'Projl' and 'Projr'
2014-02-12, by blanchet
adapted to 'xxx_{case,rec}' renaming, to new theorem names, and to new variable names in theorems
2014-02-12, by blanchet
adapted theories to 'xxx_case' to 'case_xxx'
2014-02-12, by blanchet
renamed 'nat_{case,rec}' to '{case,rec}_nat'
2014-02-12, by blanchet
renamed '{prod,sum,bool,unit}_case' to 'case_...'
2014-02-12, by blanchet
adapted theories to '{case,rec}_{list,option}' names
2014-02-12, by blanchet
avoid old 'prod.simps' -- better be more specific
2014-02-12, by blanchet
repaired hard-coded constant names
2014-02-12, by blanchet
killed 'rep_compat' option
2014-02-12, by blanchet
made 'ctr_sugar' more friendly to the 'datatype_realizer'
2014-02-12, by blanchet
use names like 'rec_mytype' and 'case_mytype' in old datatype package as well, to avoid a mixture
2014-02-12, by blanchet
use right local theory -- shows up when 'no_discs_sels' is set
2014-02-12, by blanchet
compatibility names
2014-02-12, by blanchet
use new selector support to define 'the', 'hd', 'tl'
2014-02-12, by blanchet
transformed 'option' and 'list' into new-style datatypes (but register them as old-style as well)
2014-02-12, by blanchet
avoid duplicate 'case' definitions by first looking up 'Ctr_Sugar'
2014-02-12, by blanchet
tuned code
2014-02-12, by blanchet
more 'ctr_sugar' modernization
2014-02-12, by blanchet
tuning
2014-02-12, by blanchet
ported predicate compiler to 'ctr_sugar'
2014-02-12, by blanchet
updated docs
2014-02-12, by blanchet
generate 'fundec_cong' attribute for new-style (co)datatypes
2014-02-12, by blanchet
got rid of dynamic scoping the easy way
2014-02-12, by blanchet
removed trivial 'rec' examples for nonrecursive types (I could also have added the 'old.' prefix in front of the constant names)
2014-02-12, by blanchet
more liberal merging of BNFs and constructor sugar
2014-02-12, by blanchet
se 'wrap_free_constructors' to register 'sum' , 'prod', 'unit', 'bool' with their discriminators/selectors
2014-02-12, by blanchet
have the same no-update semantics for 'case' as for 'Ctr_Sugar' and BNF data (this might not be the final word on the matter, but using a consistent policy seems like a good idea)
2014-02-12, by blanchet
Mac OS X Lion (macbroy6) is baseline for portable executables;
2014-02-11, by wenzelm
"no_memory" option for the simplifier trace to bypass memoization
2014-02-11, by Lars Hupel
tuned
2014-02-11, by nipkow
merged
2014-02-10, by wenzelm
seal system channels at end of Pure bootstrap -- Isabelle/Scala provides official interfaces;
2014-02-10, by wenzelm
make triple-sure that the future scheduler is properly shutdown (see also 702278df3b57);
2014-02-10, by wenzelm
discontinued axiomatic 'classes', 'classrel', 'arities';
2014-02-10, by wenzelm
updated keywords;
2014-02-10, by wenzelm
more explicit axiomatization;
2014-02-10, by wenzelm
prefer vacuous definitional type classes over axiomatic ones;
2014-02-10, by wenzelm
more explicit axiomatization;
2014-02-10, by wenzelm
prefer vacuous definitional type classes over axiomatic ones;
2014-02-10, by wenzelm
comments;
2014-02-10, by wenzelm
removed rotten code;
2014-02-10, by wenzelm
more elementary put_simpset: exchange the simplifier configuration outright, which is particularly relevant concerning cumulative depth, e.g. for Product_Type.split_beta in the subsequent example:
2014-02-10, by wenzelm
merged
2014-02-10, by nipkow
improved lin.arith. for terms involving division
2014-02-10, by nipkow
restoring ancient string_classes option
2014-02-09, by haftmann
method names in instance declarations are always unqualified
2014-02-09, by haftmann
dropped legacy finally
2014-02-09, by haftmann
tidied messy proofs
2014-02-09, by paulson
minimal document;
2014-02-09, by wenzelm
removed junk;
2014-02-09, by wenzelm
merged
2014-02-09, by wenzelm
check scalable fonts;
2014-02-09, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
tip