Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-3000
-1000
-960
+960
+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.
added notes;
2000-05-21, by wenzelm
new Isar version;
2000-05-21, by wenzelm
replaced {{ }} by { };
2000-05-21, by wenzelm
cite isabelle-axclass;
2000-05-21, by wenzelm
improved \BG, \EN;
2000-05-21, by wenzelm
removed is_type_abbr;
2000-05-21, by wenzelm
removed is_type_abbr;
2000-05-21, by wenzelm
adapted to inner syntax of sorts;
2000-05-21, by wenzelm
replaced {{ }} by { };
2000-05-21, by wenzelm
added sort_of_term;
2000-05-21, by wenzelm
added read_sort;
2000-05-21, by wenzelm
*** empty log message ***
2000-05-21, by wenzelm
new stuff;
2000-05-21, by wenzelm
\urlstyle{rm};
2000-05-21, by wenzelm
snapshot of new Isar'ized version;
2000-05-21, by wenzelm
added lemma.
2000-05-20, by nipkow
fixed link
2000-05-20, by nipkow
* HOL/ML: even fewer consts are declared as global (see theories Ord,
2000-05-18, by wenzelm
print_state: flag for proof only;
2000-05-18, by wenzelm
hide: check declared;
2000-05-18, by wenzelm
added disable_pr, enable_pr;
2000-05-18, by wenzelm
'pr' now prints actual proof states only;
2000-05-18, by wenzelm
fewer consts declared as global;
2000-05-18, by wenzelm
'apply' consumes facts;
2000-05-18, by wenzelm
Proof General -- if present make this the default;
2000-05-17, by wenzelm
export generic_simp_tac;
2000-05-17, by wenzelm
changed to cope with the rewriting of #2+n to Suc(Suc n)
2000-05-16, by paulson
new policy to simplify the use of numerals:
2000-05-16, by paulson
reverted to old proof of dominoes_tile_row, given new treatment of #2+...
2000-05-16, by paulson
Replaced some definitions involving epsilon by more readable primrec
2000-05-15, by berghofe
alist_rec and assoc are now defined using primrec and thus no longer
2000-05-15, by berghofe
Removed unnecessary primrec equations of hd and last involving arbitrary.
2000-05-15, by berghofe
collected three proofs into rename_client_map_tac
2000-05-15, by paulson
added the dummy theory Integ/NatSimprocs.thy
2000-05-15, by paulson
updated
2000-05-12, by paulson
new simprules needed because of new subtraction rewriting
2000-05-12, by paulson
nat_diff_split' now called nat_diff_split
2000-05-12, by paulson
deleted a lot of obsolete arithmetic lemmas
2000-05-12, by paulson
tidied
2000-05-12, by paulson
new simprules for nat_case and nat_rec
2000-05-12, by paulson
tidying, especially to remove zcompare_rls from proofs
2000-05-12, by paulson
a massive tidy-up
2000-05-12, by paulson
NatSimprocs is now a theory, not a file
2000-05-12, by paulson
new theorem one_le_power
2000-05-12, by paulson
tidied
2000-05-12, by paulson
deleted some redundant simprules
2000-05-12, by paulson
new dummy theory; prevents strange errors when loading NatSimprocs.ML
2000-05-12, by paulson
improved name of simproc;
2000-05-12, by wenzelm
fixed theory deps;
2000-05-10, by wenzelm
base on IntArith instead of Int (in order to leave out deleted simproc!);
2000-05-10, by wenzelm
dest_mss: sort procs wrt. names;
2000-05-10, by wenzelm
FAKE_BUILD;
2000-05-10, by wenzelm
polyml;
2000-05-10, by wenzelm
tuned;
2000-05-10, by wenzelm
new default simprule for better compatibility with old setup
2000-05-10, by paulson
tidied
2000-05-10, by paulson
tuned;
2000-05-10, by wenzelm
use proper version of pdfsetup.sty;
2000-05-09, by wenzelm
added semicolons;
2000-05-09, by wenzelm
updated keywords;
2000-05-09, by wenzelm
named "op ^" definitions;
2000-05-09, by wenzelm
improved X-Symbol stuff;
2000-05-09, by wenzelm
more examples
2000-05-09, by paulson
added INSTALL;
2000-05-08, by wenzelm
moved theory Sexp to Induct examples;
2000-05-08, by wenzelm
strip = impI allI allI;
2000-05-08, by wenzelm
replaced rabs by overloaded abs;
2000-05-08, by wenzelm
yet another example
2000-05-08, by paulson
new example
2000-05-08, by paulson
tidied
2000-05-08, by paulson
better simplification of the result of simprocs
2000-05-08, by paulson
moved le_square, proved le_cube
2000-05-08, by paulson
more details
2000-05-08, by paulson
tuned msg;
2000-05-08, by wenzelm
val needs_filtered_use = true;
2000-05-08, by wenzelm
recovered \seealso;
2000-05-08, by wenzelm
improved indexing;
2000-05-08, by wenzelm
\usepackage{makeidx};
2000-05-08, by wenzelm
tuned GARBAGE;
2000-05-08, by wenzelm
improved handling of Isabelle styles (less garbage);
2000-05-08, by wenzelm
updated;
2000-05-08, by wenzelm
updated syntax of simp options: (no_asm) etc.;
2000-05-08, by wenzelm
removed \isabelledefaultstyle (use \isabellestyle instead);
2000-05-08, by wenzelm
always discgarb -c;
2000-05-08, by wenzelm
fixed clash with new 'abs' const;
2000-05-06, by wenzelm
use Sign.simple_read_term;
2000-05-05, by wenzelm
error msg: counting from one (again), in order to be consistent with
2000-05-05, by wenzelm
tuned messages;
2000-05-05, by wenzelm
removed dead code: listof;
2000-05-05, by wenzelm
use Args.colon / Args.parens;
2000-05-05, by wenzelm
adapted to new arithmetic simprocs;
2000-05-05, by wenzelm
added scan_to_id (used to be in Pure/section_utils.ML);
2000-05-05, by wenzelm
removed Pure/section_utils.ML;
2000-05-05, by wenzelm
improved syntax of method options (no_asm) etc;
2000-05-05, by wenzelm
removed index2;
2000-05-05, by wenzelm
updated;
2000-05-05, by wenzelm
GPLed;
2000-05-05, by wenzelm
GPLed;
2000-05-05, by wenzelm
GPLed;
2000-05-05, by wenzelm
GPLed;
2000-05-05, by wenzelm
GPLed;
2000-05-05, by wenzelm
GPLed;
2000-05-05, by wenzelm
added simple_read_term;
2000-05-05, by wenzelm
tuned msg;
2000-05-05, by wenzelm
Added constant abs.
2000-05-05, by nipkow
simprocs now simplify the RHS of their result
2000-05-05, by paulson
new lemmas about binary division
2000-05-05, by paulson
Added AVL
2000-05-05, by nipkow
if_weak_cong should make linear arithmetic faster
2000-05-04, by paulson
a safer way of proving literal equalities
2000-05-04, by paulson
from Suc...Suc to #m
2000-05-04, by paulson
of course it should use Main
2000-05-04, by paulson
new lemmas concerning powers and #mmm
2000-05-04, by paulson
changed 2 to #2
2000-05-04, by paulson
Suc 0 -> 1
2000-05-04, by paulson
card_Pow is no longer a default simprule because it uses unary 2
2000-05-04, by paulson
simprocs
2000-05-04, by paulson
further tidying of integer simprocs
2000-05-04, by paulson
removed obsolete simproc combine_coeff
2000-05-03, by paulson
Installation of CombineNumerals for the integers
2000-05-03, by paulson
removed obsolete simprocs
2000-05-03, by paulson
removed obsolete "evenness" proofs
2000-05-02, by paulson
TEMPORARY REMOVAL OF TWO BROKEN EXAMPLES
2000-05-02, by paulson
modified for new simprocs
2000-05-02, by paulson
now using binary naturals
2000-05-02, by paulson
various bug fixes
2000-05-02, by paulson
Cassini identity is easier to prove using INTEGERS
2000-05-02, by paulson
a more modern proof
2000-05-02, by paulson
now with combine_numerals
2000-05-02, by paulson
combine_numerals replaces both fold_Suc and combine_coeff
2000-05-02, by paulson
new simproc, replacing combine_coeffs and working for nat, int, real
2000-05-02, by paulson
signature change
2000-04-28, by paulson
inserted triviality check
2000-04-28, by paulson
*** empty log message ***
2000-04-25, by nipkow
new, but still slow, proofs using binary numerals
2000-04-23, by paulson
[Int_CC.sum_conv, Int_CC.rel_conv] no longer exist
2000-04-23, by paulson
number_of now takes a type arg
2000-04-23, by paulson
this change saves 15 seconds
2000-04-23, by paulson
bug fixes to new simprocs
2000-04-23, by paulson
[Int_CC.sum_conv, Int_CC.rel_conv] no longer exist
2000-04-23, by paulson
removed some duplication, etc.
2000-04-23, by paulson
now uses the new cancel_numerals simproc
2000-04-23, by paulson
Provers/Arith/inverse_fold.ML is already obsolete
2000-04-21, by paulson
cleaner exceptions
2000-04-21, by paulson
now works for coefficients, not just for numerals
2000-04-21, by paulson
new file containing simproc invocations, from NatBin.ML
2000-04-21, by paulson
moved the simproc code to NatSimprocs.ML
2000-04-21, by paulson
Provers/Arith/inverse_fold.ML is already obsolete
2000-04-21, by paulson
new file Integ/NatSimprocs.ML
2000-04-21, by paulson
Provers/Arith/inverse_fold.ML is already obsolete
2000-04-21, by paulson
*** empty log message ***
2000-04-20, by nipkow
*** empty log message ***
2000-04-19, by nipkow
TuturialI;
2000-04-19, by wenzelm
*** empty log message ***
2000-04-19, by nipkow
check_file: keep expanded (!) absolute path;
2000-04-19, by wenzelm
Adding generated files
2000-04-19, by nipkow
*** empty log message ***
2000-04-19, by nipkow
fixed -c default value;
2000-04-19, by wenzelm
Adding generated files.
2000-04-19, by nipkow
I wonder which files i forgot.
2000-04-19, by nipkow
*** empty log message ***
2000-04-19, by nipkow
I wonder if that's all?
2000-04-19, by nipkow
deleted obsolete lemma_not_leI2
2000-04-19, by paulson
removal of less_SucI, le_SucI from default simpset
2000-04-19, by paulson
replaced obsolete diff_right_cancel by diff_diff_eq
2000-04-18, by paulson
added number_of_const: term
2000-04-18, by paulson
tidied
2000-04-18, by paulson
instantiates new simprocs for numerals of type "nat"
2000-04-18, by paulson
new simprocs for numerals of type "nat"
2000-04-18, by paulson
emilimated global names;
2000-04-18, by wenzelm
removed obsolete "simpset" keyword;
2000-04-18, by wenzelm
renamed 'hide' to 'hide_action';
2000-04-18, by wenzelm
fixed theory deps;
2000-04-18, by wenzelm
made SML/NJ happy;
2000-04-17, by wenzelm
made SML/NJ happy;
2000-04-17, by wenzelm
* improved name spaces: ambiguous output is qualified; support for
2000-04-17, by wenzelm
improved output of ambiguous entries;
2000-04-17, by wenzelm
Pretty.chunks;
2000-04-17, by wenzelm
'global' / 'local': comment;
2000-04-17, by wenzelm
name space hide operations;
2000-04-17, by wenzelm
global/local_path: comment;
2000-04-17, by wenzelm
added 'hide';
2000-04-17, by wenzelm
tuned msg;
2000-04-17, by wenzelm
NameSpace.is_qualified;
2000-04-17, by wenzelm
Pretty.chunks;
2000-04-17, by wenzelm
mod to error msg
2000-04-15, by nipkow
next_block: reset_facts;
2000-04-15, by wenzelm
plain ASCII;
2000-04-15, by wenzelm
intrn_arity: reject type abbreviations;
2000-04-14, by wenzelm
added is_type_abbr;
2000-04-14, by wenzelm
\newenvironment{isabellequote};
2000-04-14, by wenzelm
global \isa@parindent, \isa@parskip;
2000-04-14, by wenzelm
use HOLogic.termT;
2000-04-14, by wenzelm
outer syntax: no simps;
2000-04-13, by wenzelm
recdef: no simps;
2000-04-13, by wenzelm
stopped using the obsolete "nat_ind_tac"
2000-04-13, by paulson
added some new iff-lemmas; removed some obsolete thms
2000-04-13, by paulson
tidied
2000-04-13, by paulson
tuned;
2000-04-13, by wenzelm
*** empty log message ***
2000-04-13, by nipkow
Simplifier options;
2000-04-13, by wenzelm
Times -> <*>
2000-04-13, by nipkow
fixed ??/?;
2000-04-13, by wenzelm
fixed index;
2000-04-13, by wenzelm
added simp_options;
2000-04-13, by wenzelm
intro/elim_tac: match only;
2000-04-13, by wenzelm
made mod_less_divisor a simplification rule.
2000-04-13, by nipkow
InductMethod.concls_of;
2000-04-12, by wenzelm
tuned;
2000-04-12, by wenzelm
export concl_of;
2000-04-12, by wenzelm
tuned \isasymlbrace;
2000-04-12, by wenzelm
'insts' syntax;
2000-04-12, by wenzelm
improved 'induct(_tac)' syntax;
2000-04-12, by wenzelm
added 'insert' method;
2000-04-12, by wenzelm
added inst, insts;
2000-04-12, by wenzelm
improved induct_tac;
2000-04-12, by wenzelm
induct stripped: match_tac;
2000-04-12, by wenzelm
Args.name_dummy;
2000-04-12, by wenzelm
fixed 'induct_tac' syntax;
2000-04-12, by wenzelm
handle dir prefix;
2000-04-10, by wenzelm
improved document preparation;
2000-04-10, by wenzelm
fixed comment;
2000-04-08, by wenzelm
added 'ML_command';
2000-04-07, by wenzelm
apply etc.: comments;
2000-04-07, by wenzelm
tuned \isasymlbrace;
2000-04-06, by wenzelm
added \isasymlbrace, \isasymrbrace, \isasymtop;
2000-04-06, by wenzelm
'welcome' made diagnostic;
2000-04-06, by wenzelm
added Isar_examples/NestedDatatype.thy;
2000-04-05, by wenzelm
added NestedDatatype.thy;
2000-04-05, by wenzelm
added NestedDatatype;
2000-04-05, by wenzelm
fixed goal selection;
2000-04-05, by wenzelm
Isar: simplified (more robust) goal selection of proof methods;
2000-04-05, by wenzelm
induct/case_tac emulation: optional rule;
2000-04-05, by wenzelm
HEADGOAL;
2000-04-05, by wenzelm
tuned comment;
2000-04-05, by wenzelm
removed "as" keyword;
2000-04-05, by wenzelm
suppress warning;
2000-04-05, by wenzelm
print_simpset / print_claset command;
2000-04-04, by wenzelm
case_tac / induct_tac: optional rule;
2000-04-04, by wenzelm
case_tac, induct_tac;
2000-04-04, by wenzelm
'let': replaced 'as' by 'and';
2000-04-04, by wenzelm
tuned recover;
2000-04-03, by wenzelm
isapar, isamarkuptext, isamarkuptxt turned into environments;
2000-04-03, by wenzelm
markup_env_command 'text' / 'txt';
2000-04-03, by wenzelm
support markup environments;
2000-04-03, by wenzelm
tuned presentation;
2000-04-01, by wenzelm
proper naming of fib equations;
2000-04-01, by wenzelm
recdef: admit names/atts;
2000-04-01, by wenzelm
isatool document: tuned -c option;
2000-04-01, by wenzelm
recdef: admit name and atts;
2000-04-01, by wenzelm
tuned -c option;
2000-04-01, by wenzelm
recover: observe stopper;
2000-04-01, by wenzelm
presentation ignore stuff: swallow newline;
2000-04-01, by wenzelm
added is_newline;
2000-04-01, by wenzelm
'cd': diag;
2000-04-01, by wenzelm
more robust handling of explicit rules;
2000-04-01, by wenzelm
tuned mixfix syntax;
2000-04-01, by wenzelm
added ProofGeneral.undo;
2000-04-01, by wenzelm
isatool document: check output file (workaround PolyML problem with RC);
2000-04-01, by wenzelm
use cong_add_global att;
2000-03-31, by wenzelm
added cong atts;
2000-03-31, by wenzelm
added cong atts;
2000-03-31, by wenzelm
made SML/XL happy;
2000-03-31, by wenzelm
change_global/local_css move to Provers/clasimp.ML;
2000-03-31, by wenzelm
setup cong_attrib_setup;
2000-03-31, by wenzelm
added change_global/local_css;
2000-03-31, by wenzelm
added 'cong' att;
2000-03-31, by wenzelm
tuned;
2000-03-31, by wenzelm
params: preserve case names;
2000-03-31, by wenzelm
fixed indexing of elim rules;
2000-03-31, by wenzelm
use Attrib.add_del_args;
2000-03-31, by wenzelm
added add_del_args;
2000-03-31, by wenzelm
fixed goal syntax;
2000-03-31, by wenzelm
comments modified
2000-03-31, by nipkow
tuned
2000-03-31, by kleing
included new stanford mirror, mirror links now point to source directly
2000-03-31, by kleing
updated recdef
2000-03-31, by nipkow
tuned;
2000-03-30, by wenzelm
recdef
2000-03-30, by nipkow
If all termination conditions are proved automatically,
2000-03-30, by nipkow
recdef.rules -> recdef.simps
2000-03-30, by nipkow
mod in recdef allows to access the correct simpset via simpset().
2000-03-30, by nipkow
the simplification rules returned from TFL are now paired with the row they
2000-03-30, by nipkow
* Isar/Pure: local results and corresponding term bindings are now
2000-03-30, by wenzelm
support Hindley-Milner polymorphisms in results and bindings;
2000-03-30, by wenzelm
added 'moreover' and 'ultimately';
2000-03-30, by wenzelm
added \MOREOVER, \ULTIMATELY;
2000-03-30, by wenzelm
support Hindley-Milner polymorphisms in binds and facts;
2000-03-30, by wenzelm
support Hindley-Milner polymorphisms in binds and facts;
2000-03-30, by wenzelm
let_bind(_i): polymorphic version;
2000-03-30, by wenzelm
ProofContext.find_free;
2000-03-30, by wenzelm
'tactic': refer to PureIsar structure;
2000-03-30, by wenzelm
?this: support params;
2000-03-30, by wenzelm
support polymorphic Vars;
2000-03-30, by wenzelm
tuned;
2000-03-30, by wenzelm
foldl_term_types: depend on term as well;
2000-03-30, by wenzelm
read_def_cterms: use Sign.read_def_terms;
2000-03-30, by wenzelm
read_def_terms (no certify yet);
2000-03-30, by wenzelm
export update_multi;
2000-03-30, by wenzelm
added tvars_intr_list;
2000-03-30, by wenzelm
*** empty log message ***
2000-03-29, by nipkow
*** empty log message ***
2000-03-29, by nipkow
mods because of weak_case_cong -> removed Action.ML twice
2000-03-28, by nipkow
added weak_case_cong feature
2000-03-28, by nipkow
mods because of weak_case_cong
2000-03-28, by nipkow
fixed railqtoken;
2000-03-28, by wenzelm
-I option;
2000-03-28, by wenzelm
renamed 'hoare_vcg' to 'hoare';
2000-03-27, by wenzelm
tuned;
2000-03-27, by wenzelm
fixed dddot_tr;
2000-03-27, by wenzelm
rail token vs. terminal;
2000-03-27, by wenzelm
fixed term syntax;
2000-03-27, by wenzelm
tail token vs. terminal;
2000-03-27, by wenzelm
fixed \rail@tokenfont (ever used?);
2000-03-27, by wenzelm
added an order-sorted version of quickSort
2000-03-27, by paulson
simplified constant "colored"
2000-03-27, by paulson
added 'ultimately';
2000-03-26, by wenzelm
added WhileRule';
2000-03-26, by wenzelm
made SML/NJ happy;
2000-03-26, by wenzelm
tuned presentation;
2000-03-26, by wenzelm
tuned;
2000-03-26, by wenzelm
ignore_stuff;
2000-03-26, by wenzelm
tuned output;
2000-03-26, by wenzelm
!!!! = cut "Corrupted outer syntax in presentation";
2000-03-26, by wenzelm
added is_begin/end_ignore;
2000-03-26, by wenzelm
tuned targets;
2000-03-26, by wenzelm
tuned;
2000-03-25, by wenzelm
improved (anti)quote_tr(');
2000-03-25, by wenzelm
addsimprocs [record_simproc];
2000-03-25, by wenzelm
tuned antiquote_tr';
2000-03-25, by wenzelm
export updateN;
2000-03-25, by wenzelm
use abstract syntax;
2000-03-24, by wenzelm
plain ASCII;
2000-03-24, by wenzelm
arith method: HEADGOAL;
2000-03-24, by wenzelm
HOL/ex/Multiquote;
2000-03-24, by wenzelm
added HOL/ex/Multiquote.thy;
2000-03-24, by wenzelm
tuned;
2000-03-24, by wenzelm
usedir -D: update styles as well;
2000-03-24, by wenzelm
usedir -D: update styles;
2000-03-24, by wenzelm
improved dump of styles;
2000-03-24, by wenzelm
-o sty;
2000-03-24, by wenzelm
comments
2000-03-24, by nipkow
added 'moreover' command;
2000-03-23, by wenzelm
tuned output;
2000-03-23, by wenzelm
tuned spacing;
2000-03-23, by wenzelm
ex/Antiquote.thy made new-style theory;
2000-03-23, by wenzelm
now exclusively uses rtac/dtac/etac rather than the long forms
2000-03-23, by paulson
restored the MESON examples file HOL/ex/mesontest2.ML
2000-03-23, by paulson
made a proof more robust (did not like Suc_less_eq)
2000-03-22, by paulson
Suc_less_eq now with AddIffs. How could this have been overlooked?
2000-03-22, by paulson
combined finite_Int1/2 as finite_Int. Deleted the awful "lemma" from the
2000-03-22, by paulson
made more robust
2000-03-22, by paulson
tidied using new "inst" rule
2000-03-22, by paulson
tidied using new "inst" rule
2000-03-22, by paulson
new meta-rule "inst", a shorthand for read_instantiate_sg
2000-03-22, by paulson
goal_spec: [!];
2000-03-21, by wenzelm
tuned;
2000-03-21, by wenzelm
tuned;
2000-03-21, by wenzelm
tuned;
2000-03-21, by wenzelm
tuned comment;
2000-03-21, by wenzelm
help message;
2000-03-21, by wenzelm
handle general case: params and hyps of thesis;
2000-03-21, by wenzelm
soft_asm_tac: hack to norm goal;
2000-03-21, by wenzelm
proof methods: 'case_tac' / 'induct_tac';
2000-03-20, by wenzelm
tuned degenerate cases / induct;
2000-03-20, by wenzelm
added prove_goalw_cterm;
2000-03-20, by wenzelm
quick_and_dirty moved to Isar/skip_proof.ML;
2000-03-20, by wenzelm
use Args.goal_spec;
2000-03-20, by wenzelm
goal_spec;
2000-03-20, by wenzelm
ALLGOALS_RANGE superceded by Seq.INTERVAL;
2000-03-20, by wenzelm
improved support for emulating tactic scripts;
2000-03-20, by wenzelm
res_inst_tac etc.;
2000-03-20, by wenzelm
goalspec;
2000-03-20, by wenzelm
case_tac, induct_tac;
2000-03-20, by wenzelm
tactic emulation;
2000-03-20, by wenzelm
tidied
2000-03-20, by paulson
the perm_rules variable is no longer needed
2000-03-20, by paulson
tidied
2000-03-20, by paulson
replaced best_tac by force_tac, allowing some arithmetic reasoning
2000-03-20, by paulson
renamed a variable to avoid possible free/bound confusion
2000-03-20, by paulson
a possibly (?) more perspicous simprule in the "simpset" part
2000-03-20, by paulson
now based on "Main", as it should be
2000-03-20, by paulson
deleted unnecessary "simpset" part from recdef
2000-03-20, by paulson
'oops' made proper;
2000-03-18, by wenzelm
intro_classes_tac: REPEAT_ALL_NEW;
2000-03-18, by wenzelm
tuned comments;
2000-03-18, by wenzelm
tuned;
2000-03-18, by wenzelm
obtain;
2000-03-18, by wenzelm
simplified setup;
2000-03-18, by wenzelm
pure methods / atts moved here;
2000-03-18, by wenzelm
tuned;
2000-03-18, by wenzelm
obtain;
2000-03-18, by wenzelm
parskip 0pt;
2000-03-17, by wenzelm
tuned;
2000-03-17, by wenzelm
fixed theory, context typing;
2000-03-17, by wenzelm
tuned;
2000-03-17, by wenzelm
simplified Proof General setup;
2000-03-17, by wenzelm
untag: only name arg;
2000-03-17, by wenzelm
arith: "!" arg;
2000-03-17, by wenzelm
x-symbol;
2000-03-17, by wenzelm
fixed \OBTAIN;
2000-03-17, by wenzelm
fixed dep;
2000-03-17, by wenzelm
arith method: bang arg;
2000-03-17, by wenzelm
\isamarkupheader: \section;
2000-03-17, by wenzelm
generic "kill" command;
2000-03-17, by wenzelm
old_symbol_source: include header;
2000-03-17, by wenzelm
kill: include kill_proof;
2000-03-17, by wenzelm
fixed untag;
2000-03-17, by wenzelm
untag: remove all tags of given name;
2000-03-17, by wenzelm
no begin_goal marker (interferes with "latex" etc. output; useless anyway?)
2000-03-17, by wenzelm
next_block: allow in non-goal blocks as well (experimental);
2000-03-17, by wenzelm
re-ordered the theorems
2000-03-17, by paulson
better error messages, especially for multiple types
2000-03-17, by paulson
Splitter support;
2000-03-16, by wenzelm
added HOL/PreLIst.thy;
2000-03-16, by wenzelm
tuned;
2000-03-16, by wenzelm
do not change parindent/parskip;
2000-03-16, by wenzelm
Isar: splitter support; improved diagnostics;
2000-03-16, by wenzelm
Splitter support;
2000-03-16, by wenzelm
moved "cases" to generic.tex;
2000-03-16, by wenzelm
tuned;
2000-03-16, by wenzelm
Named local contexts (cases);
2000-03-16, by wenzelm
Added setup for primrec theory data.
2000-03-15, by berghofe
get_recdef now returns None instead of raising ERROR.
2000-03-15, by berghofe
Added new theory data slot for primrec equations.
2000-03-15, by berghofe
Now returns theorems with correct names in derivations.
2000-03-15, by berghofe
Eliminated store_clasimp.
2000-03-15, by berghofe
- Fixed bug in prove_casedist_thms (proof failed because of
2000-03-15, by berghofe
made SML/XL happy;
2000-03-15, by wenzelm
## -D document;
2000-03-15, by wenzelm
renamed isabelle env;
2000-03-15, by wenzelm
splitter setup;
2000-03-15, by wenzelm
clasimp: include Splitter;
2000-03-15, by wenzelm
splitter setup;
2000-03-15, by wenzelm
tuned comments;
2000-03-15, by wenzelm
include Splitter.split_modifiers;
2000-03-15, by wenzelm
added attributes, method modifiers, theory setup;
2000-03-15, by wenzelm
export change_global_ss, change_local_ss;
2000-03-15, by wenzelm
removed export_chain;
2000-03-15, by wenzelm
eliminated toplevel stack;
2000-03-15, by wenzelm
'pr': modes, optional limit;
2000-03-15, by wenzelm
pr: modes, optional limit;
2000-03-15, by wenzelm
pretty chunks;
2000-03-15, by wenzelm
tuned comment;
2000-03-15, by wenzelm
tuned comments;
2000-03-15, by wenzelm
added pretty_goals(_marker);
2000-03-15, by wenzelm
removed Pretty.spc;
2000-03-15, by wenzelm
use Pretty.str / Pretty.raw_str;
2000-03-15, by wenzelm
removed lst, strlen, strlen_real, spc, sym;
2000-03-15, by wenzelm
made links to homepages absolute, avoids trouble with relative links on the
2000-03-15, by kleing
'undo' prints state (again);
2000-03-14, by wenzelm
pr, disable_pr, enable_pr;
2000-03-14, by wenzelm
silence undo command;
2000-03-14, by wenzelm
tuned comments;
2000-03-14, by wenzelm
invoke_case: include attributes;
2000-03-14, by wenzelm
'cases' and 'induct' methods;
2000-03-14, by wenzelm
tuned 'case';
2000-03-14, by wenzelm
added 'case' command;
2000-03-14, by wenzelm
added \NEXT;
2000-03-14, by wenzelm
proper symbol_output for "xsymbols" mode;
2000-03-13, by wenzelm
replaced exhaust_tac by case_tac;
2000-03-13, by wenzelm
renamed cases_tac to case_tac;
2000-03-13, by wenzelm
case_tac now subsumes both boolean and datatype cases;
2000-03-13, by wenzelm
use cases;
2000-03-13, by wenzelm
* HOL: exhaust_tac on datatypes superceded by new case_tac;
2000-03-13, by wenzelm
renamed cases_tac to case_tac;
2000-03-13, by wenzelm
adapted to new PureThy.add_thms etc.;
2000-03-13, by wenzelm
removed cases_of;
2000-03-13, by wenzelm
adapted to new PureThy.add_thms etc.;
2000-03-13, by wenzelm
adapted to new PureThy.add_thms etc.;
2000-03-13, by wenzelm
use HOLogic.Not;
2000-03-13, by wenzelm
adapted to new PureThy.add_thms etc.;
2000-03-13, by wenzelm
adapted to new PureThy.add_thms etc.;
2000-03-13, by wenzelm
export vars_of;
2000-03-13, by wenzelm
adapted to new PureThy.add_thms etc.;
2000-03-13, by wenzelm
added Not;
2000-03-13, by wenzelm
adapted to new PureThy.add_thms etc.;
2000-03-13, by wenzelm
tuned;
2000-03-13, by wenzelm
cases: preserve order;
2000-03-13, by wenzelm
*** empty log message ***
2000-03-13, by nipkow
exhaust -> cases
2000-03-13, by nipkow
exhaust_tac -> cases_tac
2000-03-13, by nipkow
renamed "f" to "le" and "mset" to "multiset"
2000-03-13, by paulson
fixed the goal statement of sorted_qsort
2000-03-13, by paulson
adapted to new PureThy.add_thms etc.;
2000-03-13, by wenzelm
add_thms, add_axioms, add_defs: return theorems as well;
2000-03-13, by wenzelm
added |>> and |>>>;
2000-03-13, by wenzelm
exhaust->cases
2000-03-13, by nipkow
Type.typ_match now uses Vartab instead of association lists.
2000-03-10, by berghofe
tidied
2000-03-10, by paulson
now uses recdef instead of "rules"
2000-03-10, by paulson
tidied, and new thm perm_append2_eq
2000-03-10, by paulson
cases_tac
2000-03-10, by nipkow
Type.typ_match now uses Vartab instead of association lists.
2000-03-10, by berghofe
Type.unify now uses Vartab instead of association lists.
2000-03-10, by berghofe
Added function min_key.
2000-03-10, by berghofe
Added functions subst_TVars_Vartab and typ_subst_TVars_Vartab.
2000-03-10, by berghofe
Envir now uses Vartab instead of association lists.
2000-03-10, by berghofe
Type.unify and Type.typ_match now use Vartab instead of association lists.
2000-03-10, by berghofe
add_cases_induct: produce proper case names;
2000-03-10, by wenzelm
type descr;
2000-03-10, by wenzelm
check_case: disallow (T)Vars in invoked case;
2000-03-09, by wenzelm
quote tag arguments;
2000-03-09, by wenzelm
more robust case names of induct;
2000-03-09, by wenzelm
cleaned comment;
2000-03-09, by wenzelm
nicely tarted up Mutil
2000-03-09, by paulson
renamed to rsync-isabelle;
2000-03-09, by wenzelm
tuned;
2000-03-09, by wenzelm
made rsync "official"
2000-03-09, by kleing
mod_less, div_less are now default simprules
2000-03-09, by paulson
moved more lemmas to Convert (transitivity etc)
2000-03-09, by kleing
mod_less, div_less are now default simprules
2000-03-09, by paulson
Factorization
2000-03-09, by paulson
rsync goes "official" (started at boot time)
2000-03-09, by kleing
tuned for completeness of LBV
2000-03-09, by kleing
some more small lemmas
2000-03-09, by kleing
completeness of the lightweight bytecode verifier
2000-03-09, by kleing
added NT case for method invocation
2000-03-09, by kleing
minor adjustments in branch and method invocation for completeness of LBV
2000-03-09, by kleing
updated discussion of compilers
2000-03-09, by paulson
add_cases: omit unnamed;
2000-03-08, by wenzelm
invoke_case: name assumption;
2000-03-08, by wenzelm
fixed section syntax;
2000-03-08, by wenzelm
sect: exlude ":" from parser;
2000-03-08, by wenzelm
removed tune_names;
2000-03-08, by wenzelm
tuned ML types;
2000-03-08, by wenzelm
tuned;
2000-03-08, by wenzelm
added \CASE, \OBTAIN, \SORRY, \OOPS;
2000-03-08, by wenzelm
added dest_global/local_rules;
2000-03-08, by wenzelm
mk_elims, add_cases_induct: name rule cases;
2000-03-08, by wenzelm
generalized FINDGOAL, HEADGOAL;
2000-03-08, by wenzelm
handling of local contexts: print_cases, get_case, add_cases;
2000-03-08, by wenzelm
added METHOD_CASES, resolveq_cases_tac;
2000-03-08, by wenzelm
added invoke_case;
2000-03-08, by wenzelm
added 'case' command;
2000-03-08, by wenzelm
added print_cases;
2000-03-08, by wenzelm
added 'case_names' and 'params';
2000-03-08, by wenzelm
added rule_cases.ML;
2000-03-08, by wenzelm
export ALLGOALS_RANGE;
2000-03-08, by wenzelm
added (un)tag_rule;
2000-03-08, by wenzelm
added Isar/rule_cases.ML;
2000-03-08, by wenzelm
added isatool mkdir;
2000-03-08, by wenzelm
isabelle -c: tell ML system to compress output image;
2000-03-08, by wenzelm
pass -c option;
2000-03-08, by wenzelm
observe COMPRESS option;
2000-03-08, by wenzelm
option -c: tell ML system to compress output image;
2000-03-08, by wenzelm
* isatool mkdir provides easy setup of Isabelle session directories,
2000-03-08, by wenzelm
tuned error msg: rows counted from 1;
2000-03-08, by wenzelm
tidied
2000-03-08, by paulson
tidied
2000-03-08, by paulson
function "remove" and new lemmas for Factorization
2000-03-08, by paulson
new theory ex/Factorization
2000-03-08, by paulson
new lemmas
2000-03-08, by paulson
added simple_args;
2000-03-06, by wenzelm
argument: include verbatim;
2000-03-06, by wenzelm
moved use_mltext, use_mltext_theory, use_let, use_setup to context.ML;
2000-03-06, by wenzelm
added use_mltext, use_mltext_theory, use_let, use_setup (from isar_thy.ML);
2000-03-06, by wenzelm
rsyncd setup;
2000-03-06, by wenzelm
switched to mirroring with rsync server
2000-03-06, by kleing
new Poly/ML setup made default;
2000-03-06, by wenzelm
induct: "stripped" option;
2000-03-04, by wenzelm
require NatDef;
2000-03-04, by wenzelm
REPEAT_ALL_NEW;
2000-03-04, by wenzelm
added REPEAT_ALL_NEW;
2000-03-04, by wenzelm
tidied
2000-03-04, by paulson
tidied
2000-03-04, by paulson
new theories UNITY/Detects, UNITY/Reachability
2000-03-04, by paulson
added con_elim_s(olved_)tac;
2000-03-03, by wenzelm
mk_cases / inductive_cases: use InductMethod.con_elim_(solved_)tac;
2000-03-03, by wenzelm
added multi_resolveq, resolveq_tac;
2000-03-03, by wenzelm
Added Tanja's Detects and Reachability theories. Also
2000-03-03, by paulson
improved reasoning about {} and UNIV
2000-03-03, by paulson
join_rules: compatibility check;
2000-03-03, by wenzelm
token_trans: symbol length;
2000-03-03, by wenzelm
join induct rules;
2000-03-02, by wenzelm
added 'prolog' method;
2000-03-02, by wenzelm
added freeze_all;
2000-03-02, by wenzelm
polished version of the Allocator using Rename
2000-03-02, by paulson
tidied the proofs of singleton_insert_inj_eq, singleton_insert_inj_eq' and
2000-03-02, by paulson
project induct rule;
2000-03-01, by wenzelm
tuned;
2000-03-01, by wenzelm
test setup;
2000-03-01, by wenzelm
proper setup;
2000-03-01, by wenzelm
tuned;
2000-03-01, by wenzelm
expandshort
2000-03-01, by paulson
added a reference
2000-03-01, by paulson
new theorems from Sidi Ould Ehmety
2000-03-01, by paulson
tuned;
2000-02-29, by wenzelm
add_cases_induct: project_rules accomodates mutual induction;
2000-02-29, by wenzelm
tuned msgs;
2000-02-29, by wenzelm
even Alloc works again, using "rename"
2000-02-29, by paulson
replaced UN_constant, INT_constant by unconditional versions that rewrite
2000-02-29, by paulson
add_cases_induct: accomodate no_elim and no_ind flags;
2000-02-28, by wenzelm
new mostly working version; Alloc nearly converted to "Rename"
2000-02-28, by paulson
new thm vimage_Collect_eq
2000-02-28, by paulson
more bijection theorems
2000-02-28, by paulson
cases/induct attributes;
2000-02-27, by wenzelm
add_cases_induct: induct_method setup;
2000-02-27, by wenzelm
HOLogic.dest_conj;
2000-02-27, by wenzelm
HOLogic.dest_conj;
2000-02-27, by wenzelm
even better induct setup;
2000-02-27, by wenzelm
early setup of induct_method;
2000-02-27, by wenzelm
added dest_conj;
2000-02-27, by wenzelm
theorems [trans] = rev_mp mp;
2000-02-27, by wenzelm
use NetRules;
2000-02-27, by wenzelm
added major_prem_of;
2000-02-27, by wenzelm
added Isar/net_rules.ML;
2000-02-27, by wenzelm
simplified induct method;
2000-02-24, by wenzelm
tuned;
2000-02-24, by wenzelm
induct method: implicit rule;
2000-02-24, by wenzelm
rN = "record";
2000-02-24, by wenzelm
all_cases / all_inducts;
2000-02-24, by wenzelm
workaround res_inst_tac/lift_inst_rule bug by explicit type contraint;
2000-02-24, by wenzelm
capply, cabs: Sign.nodup_vars;
2000-02-24, by wenzelm
nodup_vars: fixed omission of 2 minor cases; account for Frees as well;
2000-02-24, by wenzelm
tuned generated TeX code;
2000-02-24, by wenzelm
renamed a lemma
2000-02-24, by nipkow
Added and renamed a lemma.
2000-02-24, by nipkow
not working yet. partial conversion to use "rename" instead of "extend"
2000-02-23, by paulson
new theorems inj_iff, surj_iff
2000-02-23, by paulson
new reference korf85
2000-02-23, by paulson
* Pure now provides its own version of intro/elim/dest attributes;
2000-02-22, by wenzelm
tuned syntax wrapper;
2000-02-22, by wenzelm
tuned "induct" syntax;
2000-02-22, by wenzelm
"cases" method;
2000-02-22, by wenzelm
added cases_tac;
2000-02-22, by wenzelm
induct: tuned syntax;
2000-02-22, by wenzelm
added cases_of, cases;
2000-02-22, by wenzelm
removed case_split thm binding;
2000-02-22, by wenzelm
added boolN;
2000-02-22, by wenzelm
proper variant names (admit field "r");
2000-02-22, by wenzelm
three easy new examples
2000-02-22, by paulson
tuned footnote;
2000-02-21, by wenzelm
HOL/record: fixed select-update simplification procedure to handle
2000-02-21, by wenzelm
var: skolem;
2000-02-21, by wenzelm
remove *.out;
2000-02-21, by wenzelm
renamed Univalent to univalent
2000-02-21, by oheimb
simplified some proofs
2000-02-21, by paulson
new examples that cannot be done in LEO
2000-02-21, by paulson
A few lemmas and some Adds.
2000-02-21, by nipkow
Added global let-simplification rule.
2000-02-20, by nipkow
Commenst.
2000-02-19, by nipkow
added instance declaration for finite product
2000-02-18, by oheimb
added split_eta_SetCompr, SetCompr_Sigma_eq
2000-02-18, by oheimb
added Suc_le_D
2000-02-18, by oheimb
added domI, domD
2000-02-18, by oheimb
changed precedence of function update
2000-02-18, by oheimb
installed lin arith for nat numerals.
2000-02-18, by nipkow
Rename: theory for applying a bijection over states to a UNITY program
2000-02-18, by paulson
new distributive laws
2000-02-18, by paulson
expandshort
2000-02-18, by paulson
many new theorems about inj, surj etc.
2000-02-18, by paulson
new theorem nat_diff_split'
2000-02-18, by paulson
New treatment of "guarantees" with polymorphic components and bijections.
2000-02-18, by paulson
Syntax translation functions;
2000-02-16, by wenzelm
fixed some overfull lines
2000-02-16, by paulson
a smaller point size reduces the number of overfull figures
2000-02-16, by paulson
cosmetics
2000-02-15, by kleing
fixed sel_upd simproc (less efficient, but more complete);
2000-02-15, by wenzelm
lightweight bytecode verifier with correctness proof
2000-02-15, by kleing
basic source deps;
2000-02-14, by wenzelm
easy_setup: fixed mksimps;
2000-02-14, by wenzelm
proof step: reset goal_facts;
2000-02-14, by wenzelm
mkdir -p $ISABELLE_BROWSER_INFO;
2000-02-14, by wenzelm
fixed prefer;
2000-02-14, by wenzelm
tuned msg;
2000-02-14, by wenzelm
added refine_end;
2000-02-13, by wenzelm
tuned attrib;
2000-02-13, by wenzelm
apply: observe facts;
2000-02-13, by wenzelm
prf_script commands made proper;
2000-02-13, by wenzelm
refine_end;
2000-02-13, by wenzelm
attrib: keyword_symid;
2000-02-13, by wenzelm
\isabellesimplestyle;
2000-02-10, by wenzelm
symid: include single symbolic char;
2000-02-10, by wenzelm
is_symbolic;
2000-02-10, by wenzelm
theorems [elim??] = sym;
2000-02-10, by wenzelm
added easy_setup;
2000-02-10, by wenzelm
add_judgment;
2000-02-10, by wenzelm
new thm and simprule inv_id
2000-02-10, by paulson
Cambridge-specific modifications
2000-02-10, by paulson
mirror dist page;
2000-02-09, by wenzelm
tuned;
2000-02-09, by wenzelm
mirror main page;
2000-02-09, by wenzelm
clearer "Obtaining" section
2000-02-09, by kleing
[df]rule methods;
2000-02-09, by wenzelm
document -c;
2000-02-09, by wenzelm
eliminated gif dir;
2000-02-09, by wenzelm
option -c;
2000-02-09, by wenzelm
updated the Client example
2000-02-09, by paulson
tidying: mostly spacing, but also simpler forms for Crypt_imp_OR2 & OR3_imp_OR2
2000-02-09, by paulson
new thm order_less_imp_le
2000-02-09, by paulson
(then_)tac: assert_backward;
2000-02-08, by wenzelm
added -c option (beware!);
2000-02-08, by wenzelm
rename -p to -P;
2000-02-08, by wenzelm
added forget_proof;
2000-02-08, by wenzelm
added K.qed_global;
2000-02-08, by wenzelm
omit Primes;
2000-02-08, by wenzelm
(then_)apply: prove -> prove;
2000-02-07, by wenzelm
assert_no_chain;
2000-02-07, by wenzelm
refine_no_facts: recover goal_facts;
2000-02-07, by wenzelm
tuned prefer/defer;
2000-02-07, by wenzelm
intro/elim/dest attributes: changed ! / !! flags to ? / ??;
2000-02-07, by wenzelm
paper available
2000-02-07, by oheimb
tidied some proofs
2000-02-07, by paulson
Branch: top elements of stack only need to be convertible (not equal)
2000-02-05, by kleing
tuned;
2000-02-05, by wenzelm
-I option;
2000-02-05, by wenzelm
-D PATH: dump generated document sources into PATH;
2000-02-05, by wenzelm
additional tex dump;
2000-02-05, by wenzelm
'.' == by this;
2000-02-05, by wenzelm
misc improvements;
2000-02-04, by wenzelm
added MicroJava/document;
2000-02-04, by wenzelm
added old_symbol_source;
2000-02-04, by wenzelm
Present.old_symbol_source;
2000-02-04, by wenzelm
tuned;
2000-02-04, by wenzelm
manually load session;
2000-02-04, by wenzelm
tuned syms;
2000-02-04, by wenzelm
new theorem gcd_add_mult
2000-02-04, by paulson
most_general_varify_tfrees all results;
2000-02-02, by wenzelm
Rduced Class C <= Class D to C <= D.
2000-02-02, by nipkow
nat as names;
2000-02-02, by wenzelm
expandshort
2000-02-02, by paulson
new lemma fun_cons_restrict_eq
2000-02-02, by paulson
new theorems by Sidi O. Ehmety
2000-02-02, by paulson
added forgotten definition of make_imp_tac
2000-02-01, by oheimb
added forgotten rules to make IMPP
2000-02-01, by oheimb
eliminated nonascii;
2000-02-01, by wenzelm
added IMPP to HOL
2000-01-31, by oheimb
renamed image_Union_eq -> image_Union
2000-01-31, by paulson
new theorem vimage_Union
2000-01-31, by paulson
new theorem rev_ImageI
2000-01-31, by paulson
various theorems about image and inverse image
2000-01-31, by paulson
Pi_empty1 is a more general simprule than empty_fun
2000-01-31, by paulson
rm -f *.aux;
2000-01-30, by wenzelm
simp_all method;
2000-01-29, by wenzelm
eliminated proof script;
2000-01-28, by wenzelm
HEADGOAL;
2000-01-28, by wenzelm
added prefer, defer;
2000-01-28, by wenzelm
added HEADGOAL;
2000-01-28, by wenzelm
added defer, prefer;
2000-01-28, by wenzelm
Drule.instantiate;
2000-01-28, by wenzelm
cp -r;
2000-01-28, by wenzelm
-p option;
2000-01-28, by wenzelm
added range_composition (also to simpset)
2000-01-28, by oheimb
added finite_range_updI, finite_range_map_of, finite_range_map_of_override
2000-01-28, by oheimb
mkdir: prepare logic session directory;
2000-01-28, by wenzelm
added full_nat_induct
2000-01-28, by oheimb
added splitE', also to claset
2000-01-28, by oheimb
added inj_singleton
2000-01-28, by oheimb
added finite_range_imageI
2000-01-28, by oheimb
replaced FIRSTGOAL by FINDGOAL (backtracking!);
2000-01-28, by wenzelm
maintain standard rules (beware: classical provers provides another version!);
2000-01-28, by wenzelm
replaced FIRSTGOAL by FINDGOAL (backtracking!);
2000-01-28, by wenzelm
tuned sig;
2000-01-28, by wenzelm
map data;
2000-01-28, by wenzelm
added tacticals DETERM_UNTIL and DETERM_UNTIL_SOLVED
2000-01-28, by oheimb
beautified spacing for binders with symbols syntax, analogous to HOL.thy
2000-01-28, by oheimb
*** empty log message ***
2000-01-27, by oheimb
'name' etc. include 'number';
2000-01-26, by wenzelm
'name' syntax includes numbers;
2000-01-26, by wenzelm
optimized xs[i:=x]!j lemmas.
2000-01-26, by nipkow
added map, map_st;
2000-01-25, by wenzelm
added map;
2000-01-25, by wenzelm
fallback on PureThy version;
2000-01-25, by wenzelm
replaced f : A funcset B by f``A <= B.
2000-01-25, by nipkow
reflexivity simp rules
2000-01-24, by kleing
new theorem inj_on_restrict_eq
2000-01-21, by paulson
removed Isar_examples/Minimal;
2000-01-20, by wenzelm
fixed many bad line & page breaks
2000-01-18, by paulson
Documented Thm.instantiate (not normalizing) and Drule.instantiate
2000-01-18, by paulson
www;
2000-01-17, by wenzelm
Id line inserted
2000-01-17, by kleing
changes for the makepage script in Admin
2000-01-17, by kleing
makes Isabelle main web pages
2000-01-17, by kleing
Contents: suppress comments;
2000-01-17, by wenzelm
Thm.instantiate no longer normalizes, but Drule.instantiate does
2000-01-17, by paulson
still working; a bit of polishing
2000-01-14, by paulson
new lemmas for Ntree recursor example; more simprules; more lemmas borrowed
2000-01-13, by paulson
change for new rewriting
2000-01-13, by paulson
added recursor
2000-01-13, by paulson
change in add_thmss to suppress warning
2000-01-13, by paulson
a bit of tidying
2000-01-13, by paulson
working version, with Alloc now working on the same state space as the whole
2000-01-13, by paulson
new theorem subset_Compl_self_eq
2000-01-13, by paulson
tuned comment;
2000-01-13, by wenzelm
Move some lemmas to List.
2000-01-12, by nipkow
More lemmas.
2000-01-12, by nipkow
isabellesimple: avoid paragraph;
2000-01-10, by wenzelm
int:nat->int is pushed inwards.
2000-01-10, by nipkow
Forgot to "call" MicroJava in makefile.
2000-01-10, by nipkow
tidied parentheses
2000-01-07, by paulson
tidied
2000-01-07, by paulson
new theorem leadsTo_refl and induction rule leadsTo_induct_pre
2000-01-07, by paulson
better automation for "slice"
2000-01-07, by paulson
moved some proofs from UNITY/ELT to UNITY/Project
2000-01-07, by paulson
obtain: renamed 'in' to 'where';
2000-01-06, by wenzelm
oops';
2000-01-05, by wenzelm
oops;
2000-01-05, by wenzelm
improved symbol for subcls relation
2000-01-05, by oheimb
simplified definition of appl_methds, removing m_head
2000-01-05, by oheimb
tuned;
2000-01-05, by wenzelm
obtain;
2000-01-05, by wenzelm
comment: any number of texts;
2000-01-05, by wenzelm
proof markup: any mode;
2000-01-05, by wenzelm
replaced HOLogic.termTVar by HOLogic.termT;
2000-01-05, by wenzelm
ObtainFun;
2000-01-05, by wenzelm
METHOD_CLASET': refer to *local* claset;
2000-01-05, by wenzelm
moved obtain to obtain.ML;
2000-01-05, by wenzelm
TypeInfer.logicT;
2000-01-05, by wenzelm
tuned;
2000-01-05, by wenzelm
ObtainFun;
2000-01-05, by wenzelm
added thms_ctxt_args;
2000-01-05, by wenzelm
prepare patterns only once;
2000-01-05, by wenzelm
ObtainFun;
2000-01-05, by wenzelm
present chapter;
2000-01-05, by wenzelm
removed pats;
2000-01-05, by wenzelm
chapter;
2000-01-05, by wenzelm
support for dummy variables (anyT, logicT);
2000-01-05, by wenzelm
TypeInfer.logicT;
2000-01-05, by wenzelm
new arg type for max_spec etc.
2000-01-04, by oheimb
small changes;
2000-01-03, by bauerg
removed inj_eq from the default simpset again
2000-01-03, by oheimb
removed inj_eq from the default simpset again
2000-01-03, by oheimb
removed inj_eq from the default simpset again
1999-12-23, by oheimb
updated sml package name in installation exmaple
1999-12-23, by kleing
raw_t(e)xt: any proof mode;
1999-12-22, by wenzelm
fixed error msg;
1999-12-22, by wenzelm
marg_comment: repeat;
1999-12-22, by wenzelm
text: string list;
1999-12-22, by wenzelm
tidied, with a bit more progress
1999-12-22, by paulson
Working version after a FAILED attempt to base Follows upon LeadsETo
1999-12-22, by paulson
new weakening laws
1999-12-22, by paulson
removing the "{} : CC" requirement for leadsTo[CC]
1999-12-22, by paulson
back to old sml version (due to c library problems)
1999-12-22, by kleing
some tuning (incorporated David's suggestions)
1999-12-22, by kleing
working with weak LeadsTo in guarantees precondition\!
1999-12-21, by paulson
corrected, improved eMail addresses, user interface section
1999-12-21, by oheimb
now workign as far as System_Alloc_Progress
1999-12-17, by paulson
SOUNDNESS BUG FIX for rotate_rule. The original code did not expect
1999-12-16, by paulson
first working version to Alloc/System_Client_Progress;
1999-12-15, by paulson
expandshort
1999-12-13, by paulson
dist page now in page/dist-{content|layout}
1999-12-09, by kleing
updated;
1999-12-09, by wenzelm
prettyfied
1999-12-09, by kleing
full url to local (munich) page
1999-12-09, by kleing
new web pages integrated
1999-12-09, by kleing
used for new weg page layout
1999-12-09, by kleing
ID line added
1999-12-09, by kleing
new webpage layout
1999-12-09, by kleing
abolition of localTo: instead "guarantees" has local vars as extra argument
1999-12-08, by paulson
used image_eq_UN to speed up slow proofs of base cases
1999-12-08, by paulson
useful lemma eqset_imp_iff
1999-12-08, by paulson
tuned;
1999-12-07, by wenzelm
tuned;
1999-12-07, by wenzelm
added Isar_examples/Fibonacci.thy;
1999-12-07, by wenzelm
Fixed bug in find-functions: list of parameters must be reversed before
1999-12-07, by nipkow
Renamed some vars
1999-12-06, by nipkow
cosmetic mod.
1999-12-02, by nipkow
accommodate current version of rpm;
1999-12-01, by wenzelm
Fixed a problem with returning from the last frame.
1999-12-01, by nipkow
new generalized leads-to theory
1999-12-01, by paulson
fixed the discrepancy in the ordering of the constructors LESS EQUAL GREATER
1999-12-01, by paulson
deleted rogue copy of localTo_imp_o_localTo
1999-11-30, by paulson
working version with new theory ELT
1999-11-30, by paulson
new theory UNITY/ELT
1999-11-30, by paulson
Goal: tuned pris;
1999-11-29, by wenzelm
Removed !!
1999-11-29, by nipkow
Minimal.thy;
1999-11-29, by wenzelm
Isar_examples/Minimal.thy;
1999-11-29, by wenzelm
qed "";
1999-11-29, by wenzelm
Various little changes like cmethd -> method and cfield -> field.
1999-11-26, by nipkow
del Method.ML
1999-11-25, by nipkow
Minor mods.
1999-11-25, by nipkow
renamed comp to compile (avoids clash with Relation.comp);
1999-11-24, by wenzelm
prove_goal thy;
1999-11-24, by wenzelm
Basis now Main.
1999-11-24, by nipkow
tidied, choosing nicer names
1999-11-24, by paulson
distributive laws for * over -
1999-11-23, by paulson
tidied
1999-11-23, by paulson
new theorem rev_image_eqI
1999-11-23, by paulson
Added linord_less_split
1999-11-22, by nipkow
re-shaped and re-ordered conversion relations
1999-11-19, by oheimb
Streamlined it a bit more.
1999-11-18, by nipkow
A small mod.
1999-11-18, by nipkow
added Isar_examples/Puzzle.thy;
1999-11-17, by wenzelm
tidied
1999-11-17, by paulson
Streamlined it a bit.
1999-11-15, by nipkow
removed full_SetCompr_eq from simpset() again
1999-11-12, by oheimb
Added the proof by Nielson & Nielson.
1999-11-12, by nipkow
tuned;
1999-11-12, by wenzelm
HOL changes
1999-11-11, by paulson
*** empty log message ***
1999-11-11, by nipkow
Added MicroJava
1999-11-11, by nipkow
*** empty log message ***
1999-11-11, by nipkow
with_path;
1999-11-11, by wenzelm
Imported Conny's lemmas from MicroJava
1999-11-11, by nipkow
clean target;
1999-11-11, by wenzelm
header;
1999-11-11, by wenzelm
tidied
1999-11-11, by paulson
new-style infix declaration for "image"
1999-11-11, by paulson
Fixed obsolete use of "op ^^"; new lemma
1999-11-11, by paulson
tuned;
1999-11-06, by wenzelm
tidied
1999-11-05, by paulson
new psubset lemma
1999-11-05, by paulson
added foldr
1999-11-05, by paulson
Algebra and Polynomial theories, by Clemens Ballarin
1999-11-05, by paulson
Algebra and Polynomial theories, by Clemens Ballarin
1999-11-05, by paulson
tuned;
1999-11-03, by wenzelm
MUCKE_HOME;
1999-11-03, by wenzelm
Id;
1999-11-03, by wenzelm
improved;
1999-11-03, by wenzelm
tuned;
1999-11-02, by wenzelm
RPMRELEASE;
1999-11-01, by wenzelm
inserted {...}
1999-11-01, by paulson
updated;
Isabelle99
1999-10-31, by wenzelm
updated;
1999-10-31, by wenzelm
tuned;
1999-10-31, by wenzelm
tuned;
1999-10-31, by wenzelm
Isabelle99;
1999-10-30, by wenzelm
fixed deps;
1999-10-30, by wenzelm
tuned;
1999-10-30, by wenzelm
tuned;
1999-10-30, by wenzelm
improved presentation;
1999-10-30, by wenzelm
tuned;
1999-10-30, by wenzelm
isabellesym.sty;
1999-10-30, by wenzelm
definitions of many Isabelle symbols;
1999-10-30, by wenzelm
final update by Gertrud Bauer;
1999-10-29, by wenzelm
workaround bug (feature?) in bibtex;
1999-10-29, by wenzelm
tuned;
1999-10-29, by wenzelm
comment out isabellesym.sty;
1999-10-29, by wenzelm
improved;
1999-10-29, by wenzelm
\isasymbol renamed to \isasym;
1999-10-29, by wenzelm
tuned;
1999-10-29, by wenzelm
tuned msg;
1999-10-29, by wenzelm
\isasym;
1999-10-29, by wenzelm
improved singleton_insert_inj_eq
1999-10-29, by oheimb
improved presentation;
1999-10-28, by wenzelm
fixed deps;
1999-10-28, by wenzelm
tuned;
1999-10-28, by wenzelm
expandshort; tidied
1999-10-28, by paulson
localTo_imp_o_localTo is now really an implication
1999-10-28, by paulson
simplified the stable_completion proofs
1999-10-28, by paulson
tidied
1999-10-28, by paulson
expandshort
1999-10-28, by paulson
improved IsarThy.init_context;
1999-10-28, by wenzelm
tuned;
1999-10-28, by wenzelm
added various little lemmas
1999-10-27, by oheimb
clarsimp_tac now copes with the (unwanted) case that the simplifier splits
1999-10-27, by oheimb
tuned msg;
1999-10-27, by wenzelm
tuned;
1999-10-27, by wenzelm
added (try_)update_thy_only;
1999-10-27, by wenzelm
added init_context;
1999-10-27, by wenzelm
quiet_update_thy: ml flag;
1999-10-27, by wenzelm
Fixed a bug in the EX simproc.
1999-10-27, by nipkow
export cond_with_path;
1999-10-27, by wenzelm
dummy_pattern: aprop;
1999-10-27, by wenzelm
updated for Isabelle99;
1999-10-27, by wenzelm
working again; new treatment of LocalTo
1999-10-27, by paulson
TEMPORARY use of Addsimps
1999-10-27, by paulson
got rid of split_diff, which duplicated nat_diff_split, and
1999-10-27, by paulson
less
more
|
(0)
-3000
-1000
-960
+960
+1000
+3000
+10000
+30000
tip