Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-112
+112
+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.
moved print_mode to General/output.ML; load General/pretty.ML early;
2004-05-29, by wenzelm
added Pure/General/output.ML;
2004-05-29, by wenzelm
avoid 'handle _' -- would cover Interrupt as well!!!
2004-05-29, by wenzelm
Sign.infer_types: Sign.pp;
2004-05-29, by wenzelm
Library.read_int;
2004-05-29, by wenzelm
Output.output;
2004-05-29, by wenzelm
'classrel': support multiple arguments;
2004-05-29, by wenzelm
* ML: all output via channels of writeln etc. passed through Output.output;
2004-05-29, by wenzelm
output channels;
2004-05-29, by wenzelm
added asm_lr_simplify/asm_lr_rewrite and adapted asm_full_simplify/asm_full_rewrite to match to corresponding simp_tacs
2004-05-28, by schirmer
new skolemize_tac and skolemize method
2004-05-28, by paulson
new theorem Collect_imp_eq
2004-05-28, by paulson
abstraction over functions is no default any more.
2004-05-26, by chaieb
adjusted for different signature of Type.typ_instance
2004-05-26, by webertj
mainly new/different datatype examples
2004-05-26, by webertj
documentation updated
2004-05-26, by webertj
major code change: refute can now handle any Isabelle term, adds certain axioms automatically, and can handle inductive datatypes (but not yet recursion over them)
2004-05-26, by webertj
new default parameters for refute
2004-05-26, by webertj
solver "auto" now issues a warning when it uses solver "enumerate"
2004-05-26, by webertj
Corrected printer bug for bounded quantifiers Q x<=y. P
2004-05-26, by nipkow
more group isomorphisms
2004-05-26, by paulson
added drop_take:thm
2004-05-24, by nipkow
- deleted unneeded function eta_long (now in Pure/pattern.ML
2004-05-21, by berghofe
Adapted to new syntax for case expressions.
2004-05-21, by berghofe
Added more flexible parse / print translations for case expressions.
2004-05-21, by berghofe
Modified functions pt_to_ast and ast_to_term to improve handling
2004-05-21, by berghofe
- exported result datatype
2004-05-21, by berghofe
updated;
2004-05-21, by wenzelm
Pure: clear separation of logical types and nonterminals;
2004-05-21, by wenzelm
adapted tsig/sg interface;
2004-05-21, by wenzelm
added dest, minimals, maximals, is_edge, add_edge/merge_trans_acyclic;
2004-05-21, by wenzelm
added fold, product; removed transitive_closure;
2004-05-21, by wenzelm
adapted names of some sort ops;
2004-05-21, by wenzelm
major cleanup of tsig datastructures and extend/merge operations; fixes old bugs in classes/arities code; proper treatment of nonterminals and syntax-only types;
2004-05-21, by wenzelm
Type.strip_sorts;
2004-05-21, by wenzelm
incorporate type inference interface from type.ML;
2004-05-21, by wenzelm
adapted tsig interface;
2004-05-21, by wenzelm
moved some sort ops to sorts.ML; added string_of_vname (from Syntax module);
2004-05-21, by wenzelm
test_classrel/arity improve error reporting; tuned;
2004-05-21, by wenzelm
xxx_typ_raw replace xxx_typ_no_norm forms; prevent duplicate consts declarations in merge; misc cleanup;
2004-05-21, by wenzelm
string_of_vname moved to term.ML;
2004-05-21, by wenzelm
incorporate sort ops from term.ML; use Graph.T; misc cleanup;
2004-05-21, by wenzelm
type.ML now before Syntax module;
2004-05-21, by wenzelm
xxx_typ_raw replace xxx_typ_no_norm forms;
2004-05-21, by wenzelm
'classrel' now allows multiple arguments;
2004-05-21, by wenzelm
Sign.certify_tyname;
2004-05-21, by wenzelm
TypeInfer.paramify_dummies, TypeInfer.param;
2004-05-21, by wenzelm
Args.local_typ_raw;
2004-05-21, by wenzelm
output_tym: removed duplicate clauses;
2004-05-21, by wenzelm
Graph.minimals;
2004-05-21, by wenzelm
adapted syntax to cope with lack of non-logical types;
2004-05-21, by wenzelm
Type.typ_instance;
2004-05-21, by wenzelm
load ML files only once;
2004-05-21, by wenzelm
removed duplicate thms;
2004-05-21, by wenzelm
Sign.typ_instance;
2004-05-21, by wenzelm
tuned message;
2004-05-21, by wenzelm
tuned document;
2004-05-21, by wenzelm
use plain SOME;
2004-05-21, by wenzelm
proper use of 'syntax';
2004-05-21, by wenzelm
auto update
2004-05-19, by paulson
has_consts now handles the @-operator
2004-05-19, by paulson
new bij_betw operator
2004-05-19, by paulson
more results about isomorphisms
2004-05-19, by paulson
conversion of Hilbert_Choice to Isar script
2004-05-19, by paulson
the function list1 has been exported.
2004-05-19, by chaieb
A new implementation for presburger arithmetic following the one suggested in technical report Chaieb Amine and Tobias Nipkow. It is generic an smaller.
2004-05-19, by chaieb
tactic call changed from TRYALL arith_tac to TRYALL simple_arith_tac preventing a call to presburger.
2004-05-19, by chaieb
modified abel_cancel.ML for polymorphic types
2004-05-18, by obua
simplification for abelian groups
2004-05-18, by obua
Modification / Installation of Provers/Arith/abel_cancel.ML for OrderedGroup.thy
2004-05-18, by obua
Comments fixed
2004-05-17, by webertj
lemma disjoint_int_union removed - too special
2004-05-17, by mehta
Change of theory hierarchy: Group is now based in Lattice.
2004-05-14, by ballarin
tidied
2004-05-14, by paulson
new atomize theorem
2004-05-14, by paulson
removed a premise of card_inj_on_le
2004-05-14, by paulson
removal of locale coset
2004-05-14, by paulson
deleted redundant proof lines
2004-05-14, by paulson
new lemmas
2004-05-14, by paulson
clauses for ordinary resolution
2004-05-14, by paulson
conversion of theorems to atomic form
2004-05-14, by paulson
New simp rules added:
2004-05-13, by mehta
simpilified and strengthened proofs
2004-05-12, by paulson
fixed latex problems
2004-05-12, by nipkow
renamed `> to o_m
2004-05-12, by nipkow
changes made due to new Ring_and_Field theory
2004-05-11, by obua
Eta-expanded function scan_comment to make SmlNJ happy.
2004-05-11, by berghofe
broken no longer includes TTP, and other minor changes
2004-05-11, by paulson
removal of prime characters
2004-05-11, by paulson
package needed for superscripts
2004-05-11, by paulson
conversion to clauses for ordinary resolution rather than ME
2004-05-11, by paulson
auto update
2004-05-11, by paulson
Pure: nested comments in inner syntax;
2004-05-10, by wenzelm
support nested comments;
2004-05-10, by wenzelm
changed Symbol.beginning;
2004-05-10, by wenzelm
tuned;
2004-05-10, by wenzelm
Source.of_list: no buffer limitation (now pointless due to tail-recursive Scan.repeat);
2004-05-10, by wenzelm
added Scan.list;
2004-05-10, by wenzelm
ProofGeneral.process_pgip command;
2004-05-10, by wenzelm
preparation for integration with new Ring_and_Field.thy
2004-05-10, by obua
moved first lemma in LongDiv.ML to LongDiv.thy
2004-05-10, by obua
replaced apply-style proof for instance Multiset :: plus_ac0 by recommended Isar proof style
2004-05-09, by obua
removed Aux.thy;
2004-05-09, by bauerg
cleanup up read functions, include liberal versions;
2004-05-07, by wenzelm
be liberal about constant names;
2004-05-07, by wenzelm
tuned;
2004-05-07, by wenzelm
tuned notation;
2004-05-07, by wenzelm
tuned document;
2004-05-07, by wenzelm
*** empty log message ***
2004-05-07, by bauerg
Add FIXME note re FAIL (is it fixed yet?)
2004-05-07, by aspinall
Add cdata output. Add tabs in whitespace. Write two strings instead of Library.quote.
2004-05-07, by aspinall
Add -X option to trigger PGIP interaction mode.
2004-05-07, by aspinall
less
more
|
(0)
-10000
-3000
-1000
-112
+112
+1000
+3000
+10000
+30000
tip