Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-240
+240
+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 add_cnstrt
2001-10-31, by berghofe
Removed name_thm from finish_global.
2001-10-31, by berghofe
Tuned function thm_proof.
2001-10-31, by berghofe
- enter_thmx -> enter_thms
2001-10-31, by berghofe
norm_hhf_eq is now stored using open_store_standard_thm.
2001-10-31, by berghofe
induct: internalize ``missing'' consumes-facts from goal state
2001-10-31, by wenzelm
- 'induct' may now use elim-style induction rules without chaining
2001-10-31, by wenzelm
(induct set: ...);
2001-10-31, by wenzelm
put_consumes: really overwrite existing tag;
2001-10-31, by wenzelm
finish_global: Tactic.norm_hhf;
2001-10-31, by wenzelm
use HOL.induct_XXX;
2001-10-31, by wenzelm
use induct_rulify2;
2001-10-31, by wenzelm
renamed inductive_XXX to induct_XXX;
2001-10-31, by wenzelm
induct_impliesI;
2001-10-31, by wenzelm
tuned induct proofs;
2001-10-30, by wenzelm
- 'induct' method now derives symbolic cases from the *rulified* rule
2001-10-30, by wenzelm
tuned;
2001-10-30, by wenzelm
induct: cases are extracted from rulified rule;
2001-10-30, by wenzelm
removed obsolete make_raw;
2001-10-30, by wenzelm
lemma Least_mono moved from Typedef.thy to Set.thy;
2001-10-30, by wenzelm
tuned;
2001-10-29, by wenzelm
removed option -depend (not available everywhere?);
2001-10-29, by wenzelm
converted theory "Set";
2001-10-28, by wenzelm
fixed string_of_mixfix;
2001-10-28, by wenzelm
tuned declaration of rules;
2001-10-28, by wenzelm
equal_intr_rule already declared in Pure;
2001-10-28, by wenzelm
rules for meta-level conjunction;
2001-10-28, by wenzelm
tuned prove;
2001-10-28, by wenzelm
tuned;
2001-10-27, by wenzelm
added prove;
2001-10-27, by wenzelm
declare equal_intr_rule as intro;
2001-10-27, by wenzelm
tuned prove;
2001-10-27, by wenzelm
removed obsolete goal_subclass, goal_arity;
2001-10-27, by wenzelm
use Tactic.prove;
2001-10-27, by wenzelm
use Tactic.prove;
2001-10-27, by wenzelm
tuned;
2001-10-27, by wenzelm
* Pure/axclass: removed obsolete ML interface goal_subclass/goal_arity;
2001-10-27, by wenzelm
updated;
2001-10-27, by wenzelm
impose hyps on initial goal configuration (prevents res_inst_tac problems);
2001-10-27, by wenzelm
added "atomize" method;
2001-10-27, by wenzelm
prove: primitive goal interface for internal use;
2001-10-27, by wenzelm
added impose_hyps;
2001-10-27, by wenzelm
exclude field_simps from user-level "simps";
2001-10-27, by wenzelm
Isar: fixed rep_datatype args;
2001-10-27, by wenzelm
hardwire qualified const names;
2001-10-27, by wenzelm
removed "more" class;
2001-10-27, by wenzelm
moved product cases/induct to theory Datatype;
2001-10-27, by wenzelm
made new-style theory;
2001-10-27, by wenzelm
atomize_conj;
2001-10-26, by wenzelm
* Pure: method 'atomize' presents local goal premises as object-level
2001-10-26, by wenzelm
Fixed several bugs concerning arbitrarily branching datatypes.
2001-10-26, by berghofe
Eliminated occurrence of rule_format.
2001-10-26, by berghofe
tuned;
2001-10-26, by wenzelm
need at least 3 latex runs to get toc right!
2001-10-26, by wenzelm
tuned;
2001-10-26, by wenzelm
tuned;
2001-10-26, by wenzelm
Rrightarrow;
2001-10-26, by wenzelm
tuned notation;
2001-10-26, by wenzelm
tuned notation;
2001-10-26, by wenzelm
accomodate some recent changes of record package;
2001-10-25, by wenzelm
updated;
2001-10-25, by wenzelm
removed "more" sort;
2001-10-25, by wenzelm
updated records;
2001-10-25, by wenzelm
'simplified' att: args;
2001-10-25, by wenzelm
* HOL/record:
2001-10-25, by wenzelm
* Provers: 'simplified' attribute may refer to explicit rules instead
2001-10-25, by wenzelm
Replaced main proof by proper Isar script.
2001-10-25, by berghofe
derived operations are now: make, extend, truncate (cf. derived_defs);
2001-10-25, by wenzelm
tuned;
2001-10-25, by wenzelm
check_goal: setmp proofs 0;
2001-10-25, by wenzelm
added windowlistener (can now close the frame by window controls)
2001-10-25, by kleing
* HOL/record:
2001-10-25, by wenzelm
innermost_params;
2001-10-25, by wenzelm
(simp add: point.make_def);
2001-10-25, by wenzelm
provodes induct/cases for use with corresponding Isar methods;
2001-10-25, by wenzelm
further 1.73 changes: added fix_direct, simplified assume interface;
2001-10-24, by wenzelm
added read_prop_schematic;
2001-10-24, by wenzelm
simplified ProofContext.assume interface;
2001-10-24, by wenzelm
moved lambda to Pure/term.ML;
2001-10-24, by wenzelm
added lambda;
2001-10-24, by wenzelm
* clasimp: ``iff'' declarations now handle conditional rules as well;
2001-10-24, by wenzelm
added string_of_mixfix;
2001-10-24, by wenzelm
print_depth 8 from the very beginning;
2001-10-24, by wenzelm
added export_assume, export_presume, export_def (from proof.ML);
2001-10-23, by wenzelm
moved RANGE to tctical.ML;
2001-10-23, by wenzelm
added RANGE (from Isar/proof.ML);
2001-10-23, by wenzelm
print fixed names as plain strings;
2001-10-23, by wenzelm
eliminated old numerals;
2001-10-23, by wenzelm
use generic 1 instead of Numeral1;
2001-10-23, by wenzelm
eliminated Numeral0;
2001-10-23, by wenzelm
build option enables most basic browser info (for proper recording of session);
2001-10-23, by wenzelm
build option;
2001-10-23, by wenzelm
tuned;
2001-10-23, by wenzelm
eliminated old numerals;
2001-10-23, by wenzelm
pass build mode to process;
2001-10-23, by wenzelm
removed export_thm;
2001-10-23, by wenzelm
trace_rules: only non-empty;
2001-10-23, by wenzelm
removed obsolete "exported" att;
2001-10-23, by wenzelm
replace_dummy_patterns: lift over bounds;
2001-10-23, by wenzelm
iff: always rotate prems;
2001-10-23, by wenzelm
apply(simp add: three_def numerals) (* FIXME !? *);
2001-10-23, by wenzelm
unset DISPLAY (again);
2001-10-23, by wenzelm
* Pure: removed obsolete 'exported' attribute;
2001-10-23, by wenzelm
*** empty log message ***
2001-10-22, by wenzelm
moved object_logic.ML to Isar/object_logic.ML;
2001-10-22, by wenzelm
moved locale.ML to Isar/locale.ML;
2001-10-22, by wenzelm
moved goal related stuff to goals.ML;
2001-10-22, by wenzelm
Display.current_goals_markers;
2001-10-22, by wenzelm
tuned;
2001-10-22, by wenzelm
moved prove_goalw_cterm to goals.ML;
2001-10-22, by wenzelm
moved local defs to proof.ML (for locales);
2001-10-22, by wenzelm
improved source arrangement of obtain;
2001-10-22, by wenzelm
rearrange sources for locales;
2001-10-22, by wenzelm
Display.print_current_goals_fn;
2001-10-22, by wenzelm
Display.print_goals;
2001-10-22, by wenzelm
Display.pretty_thms;
2001-10-22, by wenzelm
qualified names;
2001-10-22, by wenzelm
make this module appeat late in Pure;
2001-10-22, by wenzelm
print_goals stuff is back (from locale.ML);
2001-10-22, by wenzelm
reorganize sources to accomodate locales;
2001-10-22, by wenzelm
corollary;
2001-10-22, by wenzelm
quick_and_dirty_prove_goalw_cterm;
2001-10-22, by wenzelm
javac -depend;
2001-10-22, by wenzelm
-D generated;
2001-10-22, by wenzelm
Added "clean" target.
2001-10-22, by berghofe
Fixed problem with batch mode layout, which caused an AWT exception when
2001-10-22, by berghofe
initBrowser now has additional noAWT argument.
2001-10-22, by berghofe
Constructor no longer takes font as an argument.
2001-10-22, by berghofe
Moved font settings from TreeNode to TreeBrowser.
2001-10-22, by berghofe
Moved font settings from Vertex to GraphView.
2001-10-22, by berghofe
deleted the redundant first argument of adjust(a,b)
2001-10-22, by paulson
Numerals now work for the integers: the binary numerals for 0 and 1 rewrite
2001-10-22, by paulson
New simproc, needed to cope with combinations of (abstract) 0, (abstract) 1,
2001-10-22, by paulson
Numerals now work for the integers: the binary numerals for 0 and 1 rewrite
2001-10-22, by paulson
keep DISPLAY;
2001-10-22, by wenzelm
updated;
2001-10-21, by wenzelm
renamed to Typedefs.thy to avoid conflict with main HOL version;
2001-10-21, by wenzelm
* proper spacing of consecutive markup elements, especially text
2001-10-21, by wenzelm
\newif\ifisamarkup controls spacing of isabeginpar;
2001-10-21, by wenzelm
improved spacing;
2001-10-21, by wenzelm
maintain Latex.flag_markup;
2001-10-21, by wenzelm
flag_markup;
2001-10-21, by wenzelm
Types/document/Typedefs;
2001-10-21, by wenzelm
renamed Typedef.thy to Typedefs.thy (former already present in main HOL);
2001-10-21, by wenzelm
got rid of separate root.tex;
2001-10-20, by wenzelm
graceful interpretation of -i/-d/-D options;
2001-10-20, by wenzelm
include document graph;
2001-10-20, by wenzelm
document graph option;
2001-10-20, by wenzelm
conditional: bool -> (unit -> unit) -> unit;
2001-10-20, by wenzelm
added TextIO.stdErr;
2001-10-20, by wenzelm
include document graph;
2001-10-20, by wenzelm
document graphs for several sessions;
2001-10-20, by wenzelm
tuned;
2001-10-20, by wenzelm
calculational rules moved from FOL to IFOL;
2001-10-20, by wenzelm
option -g for document graph;
2001-10-20, by wenzelm
option -q also excludes -v true in generated stuff;
2001-10-20, by wenzelm
dvips -q;
2001-10-20, by wenzelm
removed -v option (handled by isabelle process);
2001-10-20, by wenzelm
-o pdf: produce *both* eps and pdf;
2001-10-20, by wenzelm
* greatly simplified document preparation setup, including more
2001-10-20, by wenzelm
got rid of ML proof scripts;
2001-10-19, by wenzelm
induct_method.ML -- proof by cases and induction on sets and types (Isar);
2001-10-19, by wenzelm
latex output: bold lambda;
2001-10-19, by wenzelm
got rid of ML proof scripts for Product_Type;
2001-10-19, by wenzelm
got rid of Provers/split_paired_all.ML;
2001-10-19, by wenzelm
improved default dependencies;
2001-10-19, by wenzelm
revert to proper version (!);
2001-10-19, by wenzelm
GPLed;
2001-10-18, by wenzelm
tuned;
2001-10-18, by wenzelm
use abstract product type instead of datatype;
2001-10-18, by wenzelm
moved atomize stuff to theory HOL;
2001-10-18, by wenzelm
legacy interfaces for axclass instantiation;
2001-10-18, by wenzelm
added map_base;
2001-10-18, by wenzelm
sane internal interfaces for instance;
2001-10-18, by wenzelm
sane internal interface for add_typedef(_i);
2001-10-18, by wenzelm
proper setup for abstract product types;
2001-10-18, by wenzelm
moved InductMethod.setup to theory HOL;
2001-10-18, by wenzelm
setup generic cases and induction (from Inductive.thy);
2001-10-18, by wenzelm
guillemot syntax;
2001-10-17, by wenzelm
improved internal interface of typedef;
2001-10-17, by wenzelm
abstract product types;
2001-10-17, by wenzelm
proper proof of split_paired_all (presently unused);
2001-10-17, by wenzelm
tuned comments;
2001-10-17, by wenzelm
added mk_UNIV;
2001-10-17, by wenzelm
tuned;
2001-10-17, by wenzelm
simplified exporter interface;
2001-10-16, by wenzelm
added implies_intr_goals;
2001-10-16, by wenzelm
tuned;
2001-10-16, by wenzelm
Tuned.
2001-10-16, by berghofe
Removed exit command from end of main method.
2001-10-16, by berghofe
PS method now calculates layout using default font metrics.
2001-10-16, by berghofe
Inserted table for character widths.
2001-10-16, by berghofe
tuned induction proofs;
2001-10-16, by wenzelm
dest_env: norm_term on rhs;
2001-10-16, by wenzelm
typedef: export result;
2001-10-16, by wenzelm
ignore typedef result;
2001-10-16, by wenzelm
declare projected induction rules stemming from nested recursion;
2001-10-16, by wenzelm
TypedefPackage.add_typedef_no_result;
2001-10-16, by wenzelm
tuned;
2001-10-16, by wenzelm
* HOL: concrete setsum syntax "\<Sum>i:A. b" == "setsum (%i. b) A"
2001-10-16, by wenzelm
option -o FILE --output to FILE (ps, eps, pdf);
2001-10-16, by wenzelm
ISABELLE_EPSTOPDF="epstopdf";
2001-10-16, by wenzelm
Font metrics used for batch mode layout (without X11 connection).
2001-10-16, by berghofe
Added support for batch mode layout (without X11 connection).
2001-10-16, by berghofe
tuned;
2001-10-16, by wenzelm
improved induct;
2001-10-16, by wenzelm
be more careful about token class markers;
2001-10-16, by wenzelm
proper order of kind names;
2001-10-16, by wenzelm
support impromptu terminology of cases parameters;
2001-10-16, by wenzelm
parser for underscore (actually a symbolic identifier!);
2001-10-16, by wenzelm
allow empty set/type name;
2001-10-16, by wenzelm
simplified resolveq_cases_tac for cases, separate version for induct;
2001-10-16, by wenzelm
tuned;
2001-10-16, by wenzelm
canonical 'cases'/'induct' rules for n-tuples (n=3..7)
2001-10-15, by kleing
canonical 'cases'/'induct' rules for n-tuples (n=3..7)
2001-10-15, by kleing
setsum syntax;
2001-10-15, by wenzelm
intro! and elim! rules;
2001-10-15, by wenzelm
tuned NetRules;
2001-10-15, by wenzelm
Tactic.orderlist;
2001-10-15, by wenzelm
ObjectLogic.rulify;
2001-10-15, by wenzelm
Tactic.rewrite_cterm;
2001-10-15, by wenzelm
GPLed;
2001-10-15, by wenzelm
ring instead of ringS;
2001-10-15, by wenzelm
ring includes plus_ac0;
2001-10-15, by wenzelm
tuned;
2001-10-15, by wenzelm
support weight;
2001-10-15, by wenzelm
bang_args;
2001-10-15, by wenzelm
qualify some names;
2001-10-15, by wenzelm
map_nth_elem;
2001-10-15, by wenzelm
renamed reset_locs to del_locs
2001-10-15, by oheimb
moved rulify to ObjectLogic;
2001-10-14, by wenzelm
moved rulify to ObjectLogic;
2001-10-14, by wenzelm
added qed_spec_mp etc.;
2001-10-14, by wenzelm
unified rewrite/rewrite_cterm/simplify interface;
2001-10-14, by wenzelm
tuned rewrite/simplify interface;
2001-10-14, by wenzelm
improved atomize setup;
2001-10-14, by wenzelm
atomize_tac etc. moved to object_logic.ML;
2001-10-14, by wenzelm
use ObjectLogic;
2001-10-14, by wenzelm
added 'atomize' attribute;
2001-10-14, by wenzelm
tuned full_rewrite;
2001-10-14, by wenzelm
less
more
|
(0)
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip