Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+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.
tuned whitespace -- recover basic Isabelle conventions;
2009-09-29, by wenzelm
merged
2009-09-29, by wenzelm
Merge with isabelle dev changes.
2009-09-29, by Thomas Sewell
Replace OldTerm.term_vars with Term.add_vars in named_cterm_instantiate.
2009-09-29, by Thomas Sewell
Avoid a possible variable name conflict in instantiating a theorem.
2009-09-28, by Thomas Sewell
Fix unescaped expressions breaking latex output in Record.thy
2009-09-28, by Thomas Sewell
Merge record patch with updates from isabelle mainline.
2009-09-28, by Thomas Sewell
Avoid record-inner constants in polymorphic definitions in Bali
2009-09-25, by Thomas Sewell
Merge with changes from isabelle dev repository.
2009-09-24, by Thomas Sewell
Initial response to feedback from Norbert, Makarius on record patch
2009-09-23, by tsewell
Branch merge for isabelle mainline updates.
2009-09-22, by Thomas Sewell
Branch merge with updates from mainline isabelle.
2009-09-17, by Thomas Sewell
Implement previous fix (don't duplicate ext_def) correctly.
2009-09-11, by Thomas Sewell
There's no particular reason to duplicate the extension
2009-09-11, by Thomas Sewell
Merged with mainline changes.
2009-09-11, by Thomas Sewell
Adjust some documentation.
2009-09-11, by Thomas Sewell
Simplification of various aspects of the IsTuple component
2009-09-10, by Thomas Sewell
Record patch imported and working.
2009-09-10, by Thomas Sewell
Initial attempt at porting record update to repository Isabelle.
2009-08-27, by tsewell
Synchronized and Unsynchronized;
2009-09-29, by wenzelm
hide "ref" by default, to enforce excplicit indication as Unsynchronized;
2009-09-29, by wenzelm
explicit indication of Unsynchronized.ref;
2009-09-29, by wenzelm
open_unsynchronized for interactive Isar loop;
2009-09-29, by wenzelm
explicit indication of Unsynchronized.ref;
2009-09-29, by wenzelm
Raw ML references as unsynchronized state variables.
2009-09-29, by wenzelm
Dummy version of state variables -- plain refs for sequential access.
2009-09-28, by wenzelm
reactivated at-sml-dev-e;
2009-09-28, by wenzelm
misc tuning and modernization;
2009-09-28, by wenzelm
moved generic cong_tac from HOL/Tools/datatype_aux.ML to Tools/cong_tac.ML, proper subgoal selection (failure, not exception);
2009-09-28, by wenzelm
merged
2009-09-28, by wenzelm
less auxiliary functions
2009-09-28, by haftmann
tuned
2009-09-28, by haftmann
shared code between rep_datatype and datatype
2009-09-28, by haftmann
further unification of datatype and rep_datatype
2009-09-28, by haftmann
avoid compound fields in datatype info record
2009-09-28, by haftmann
fold_body_thms: pass pthm identifier;
2009-09-28, by wenzelm
tuned internal source structure;
2009-09-28, by wenzelm
added fork_deps_pri;
2009-09-28, by wenzelm
merged
2009-09-28, by haftmann
explicit pointless checkpoint
2009-09-28, by haftmann
emerging common infrastructure for datatype and rep_datatype
2009-09-27, by haftmann
streamlined rep_datatype further
2009-09-27, by haftmann
simplified rep_datatype
2009-09-27, by haftmann
more appropriate order of field in dt_info
2009-09-27, by haftmann
re-established reasonable inner outline for module
2009-09-27, by haftmann
merged
2009-09-27, by wenzelm
adjusted to changes in datatype package
2009-09-27, by haftmann
merged
2009-09-27, by haftmann
dropped dead code
2009-09-27, by haftmann
registering split rules and projected induction rules; ML identifiers more close to Isar theorem names
2009-09-27, by haftmann
fold_body_thms/join_bodies: explicitly check for cyclic theorem references;
2009-09-27, by wenzelm
tuned;
2009-09-27, by wenzelm
reachable: recovered reverse post-order (lost in 73ad4884441f), which is expected for all_preds/all_succs and required for topological_order;
2009-09-27, by wenzelm
merged
2009-09-25, by paulson
New lemmas involving the real numbers, especially limits and series
2009-09-25, by paulson
NEWS; corrected spelling
2009-09-25, by haftmann
merged
2009-09-25, by haftmann
simplified proof
2009-09-23, by haftmann
removed potentially dangerous rules from pred_set_conv
2009-09-23, by haftmann
explicitly hide empty, inter, union
2009-09-23, by haftmann
merged
2009-09-23, by haftmann
merged
2009-09-23, by haftmann
merged
2009-09-23, by haftmann
inf/sup_absorb are no default simp rules any longer
2009-09-23, by haftmann
merged
2009-09-22, by haftmann
merged
2009-09-21, by haftmann
adapted proof
2009-09-21, by haftmann
merged
2009-09-21, by haftmann
tuned proofs
2009-09-21, by haftmann
tuned header
2009-09-21, by haftmann
added note on simp rules
2009-09-21, by haftmann
merged
2009-09-21, by haftmann
tuned proof; tuned headers
2009-09-21, by haftmann
merged
2009-09-21, by haftmann
tuned proofs; be more cautios wrt. default simp rules
2009-09-21, by haftmann
merged
2009-09-21, by haftmann
tuned proofs
2009-09-21, by haftmann
merged
2009-09-19, by haftmann
inter and union are mere abbreviations for inf and sup
2009-09-19, by haftmann
merged
2009-09-24, by haftmann
lemma relating fold1 and foldl; code_unfold rules for Inf_fin, Sup_fin, Min, Max, Inf, Sup
2009-09-24, by haftmann
subsumed by more general setup in List.thy
2009-09-24, by haftmann
idempotency case for fold1
2009-09-24, by haftmann
added dual for complete lattice
2009-09-24, by haftmann
merged
2009-09-24, by nipkow
record how many "proof"s are solved by s/h
2009-09-24, by nipkow
added quotes for filenames;
2009-09-24, by boehmes
merged; adopted to changes from Code_Evaluation in the predicate compiler
2009-09-24, by bulwahn
replaced sorry by oops; removed old debug functions in predicate compiler
2009-09-23, by bulwahn
added first version of quickcheck based on the predicate compiler; added a few quickcheck examples
2009-09-23, by bulwahn
adapted configuration for DatatypeCase.make_case
2009-09-23, by bulwahn
added a new example for the predicate compiler
2009-09-23, by bulwahn
added context free grammar example; removed dead code; adapted to work without quick and dirty mode; fixed typo
2009-09-23, by bulwahn
added first prototype of the extended predicate compiler
2009-09-23, by bulwahn
moved predicate compiler to Tools
2009-09-23, by bulwahn
removed generation of strange tuple modes in predicate compiler
2009-09-23, by bulwahn
extending predicate compiler and proof procedure to support tuples; testing predicate wirh HOL-MicroJava semantics
2009-09-23, by bulwahn
modified predicate compiler further to support tuples
2009-09-23, by bulwahn
changed preprocessing due to problems with LightweightJava; added transfer of thereoms; changed the type of mode to support tuples in the predicate compiler
2009-09-23, by bulwahn
handling of definitions
2009-09-23, by bulwahn
experimenting to add some useful interface for definitions
2009-09-23, by bulwahn
added predicate compile preprocessing structure for definitional thms -- probably is replaced by hooking the theorem command differently
2009-09-23, by bulwahn
modified handling of side conditions in proof procedure of predicate compiler
2009-09-23, by bulwahn
merged
2009-09-23, by haftmann
Code_Eval(uation)
2009-09-23, by haftmann
merged
2009-09-23, by blanchet
Added "nitpick_const_simp" tags to lazy list theories.
2009-09-23, by blanchet
atbroy101 is long dead, use atbroy99; comment out broken SML test invocation
2009-09-23, by krauss
merged
2009-09-23, by haftmann
stripped legacy ML bindings
2009-09-23, by haftmann
Undo errornous commit of Statespace change
2009-09-23, by hoelzl
correct variable order in approximate-method
2009-09-23, by hoelzl
merged
2009-09-23, by paulson
Correct chasing of type variable instantiations during type unification.
2009-09-23, by paulson
hide newly introduced constants
2009-09-23, by haftmann
used standard fold function and type aliases
2009-09-22, by Philipp Meyer
sos method generates and uses proof certificates
2009-09-21, by Philipp Meyer
full reserve of worker threads -- for improved CPU utilization;
2009-09-22, by wenzelm
merged
2009-09-22, by haftmann
be more cautious wrt. simp rules: inf_absorb1, inf_absorb2, sup_absorb1, sup_absorb2 are no simp rules by default any longer
2009-09-22, by haftmann
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip