Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-3000
-1000
-480
+480
+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
less
more
|
(0)
-3000
-1000
-480
+480
+1000
+3000
+10000
+30000
tip