Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-384
+384
+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;
2007-08-02, by wenzelm
converted Meson tests to proper theory;
2007-08-02, by wenzelm
turned simp_depth_limit into configuration option;
2007-08-02, by wenzelm
added name_of;
2007-08-02, by wenzelm
turned simp_depth_limit into configuration option;
2007-08-02, by wenzelm
tuned ML bindings (for multithreading);
2007-08-01, by wenzelm
tuned ML bindings (for multithreading);
2007-08-01, by wenzelm
fix looping when applied to standard subgoals
2007-08-01, by huffman
updated;
2007-08-01, by wenzelm
tracing: level;
2007-08-01, by wenzelm
multithreading trace: int;
2007-08-01, by wenzelm
added toplevel print command;
2007-08-01, by wenzelm
tuned;
2007-08-01, by wenzelm
renamed 'print_options' to 'print_configs';
2007-08-01, by wenzelm
renamed config_option.ML to config.ML;
2007-08-01, by wenzelm
renamed config_option.ML to config.ML;
2007-08-01, by wenzelm
simplified internal Config interface;
2007-08-01, by wenzelm
updated;
2007-08-01, by wenzelm
tuned config options: eliminated separate attribute "option";
2007-08-01, by wenzelm
oops -- fixed syntax;
2007-08-01, by wenzelm
"running": PROTECTED wakeup;
2007-08-01, by wenzelm
proper path specifications;
2007-07-31, by wenzelm
simultaneous use_thys;
2007-07-31, by wenzelm
setmp_noncritical print_mode;
2007-07-31, by wenzelm
simultaneous use_thys;
2007-07-31, by wenzelm
removed obsolete HOL/Real/ROOT.ML;
2007-07-31, by wenzelm
no_document: setmp_noncritical;
2007-07-31, by wenzelm
with_charset: setmp_noncritical;
2007-07-31, by wenzelm
added max-threads preference;
2007-07-31, by wenzelm
replaced depth_limit ref by blast_depth_limit configuration option;
2007-07-31, by wenzelm
replaced dtK ref by datatype_distinctness_limit configuration option;
2007-07-31, by wenzelm
moved classical tools from theory IFOL to FOL;
2007-07-31, by wenzelm
register_thy: more sanity checks;
2007-07-31, by wenzelm
moved lin_arith stuff to Tools/lin_arith.ML;
2007-07-31, by wenzelm
proper context for cooper_tac within arith;
2007-07-31, by wenzelm
tuned LinArith setup;
2007-07-31, by wenzelm
HOL setup for linear arithmetic -- moved here from arith_data.ML;
2007-07-31, by wenzelm
added Tools/lin_arith.ML;
2007-07-31, by wenzelm
tuned;
2007-07-31, by wenzelm
tuned section "Style";
2007-07-31, by wenzelm
undo a change in last commit : give a single name to the inversion lemmas for the same inductive type
2007-07-31, by narboux
Proper interpretation of total orders in lattices.
2007-07-31, by ballarin
* Configuration options;
2007-07-31, by wenzelm
added configuration options;
2007-07-31, by wenzelm
removed use/update_thy_only;
2007-07-31, by wenzelm
find_body goes under meta-quantifier ; tactic generalizes free variables;
2007-07-31, by chaieb
Added dependency on langford files in Tools/Qelim
2007-07-31, by chaieb
Tuned document
2007-07-31, by chaieb
added register_thy (replaces pretend_use_thy_only and really flag);
2007-07-31, by wenzelm
ThyInfo.register_thy;
2007-07-31, by wenzelm
turned fast_arith_split/neq_limit into configuration options;
2007-07-31, by wenzelm
added global config options;
2007-07-31, by wenzelm
arith method setup: proper context;
2007-07-31, by wenzelm
arith method setup: proper context;
2007-07-31, by wenzelm
tuned ML declarations;
2007-07-30, by wenzelm
simultaneous use_thys;
2007-07-30, by wenzelm
dequeue: wait loop while PROTECTED -- avoids race condition;
2007-07-30, by wenzelm
marked some CRITICAL sections;
2007-07-30, by wenzelm
updated some of the definitions and proofs
2007-07-30, by urbanc
tuned msgs;
2007-07-29, by wenzelm
deps: keep thy source text, avoid reloading;
2007-07-29, by wenzelm
adapted ThyLoad.deps_thy;
2007-07-29, by wenzelm
more informative tracing;
2007-07-29, by wenzelm
load_thy: avoid reloading of text;
2007-07-29, by wenzelm
added of_list_limited (with limit argument);
2007-07-29, by wenzelm
more informative tracing;
2007-07-29, by wenzelm
explicit global state argument -- no longer CRITICAL;
2007-07-29, by wenzelm
added option -T (multithreading trace mode);
2007-07-29, by wenzelm
critical: improved diagostics;
2007-07-29, by wenzelm
tuned msg;
2007-07-29, by wenzelm
NAMED_CRITICAL;
2007-07-29, by wenzelm
removed obsolete Output.ML_errors/toplevel_errors;
2007-07-29, by wenzelm
removed obsolete Output.ML_errors/toplevel_errors;
2007-07-29, by wenzelm
added TOPLEVEL_ERROR (simplified version from output.ML);
2007-07-29, by wenzelm
removed obsolete TOPLEVEL_ERROR etc. (cf. toplevel.ML);
2007-07-29, by wenzelm
added ML toplevel use commands: Toplevel.program;
2007-07-29, by wenzelm
removed obsolete install_pp.ML (cf. pure_setup.ML);
2007-07-29, by wenzelm
replaced program_defs_ref by proper context data (via attribute "program");
2007-07-29, by wenzelm
renamed Drule.is_dummy_thm to Thm.is_dummy;
2007-07-29, by wenzelm
added list update;
2007-07-29, by wenzelm
moved Drule.add/del/merge_rules to Thm.add/del/merge_thms;
2007-07-29, by wenzelm
Named collections of theorems in canonical order.
2007-07-29, by wenzelm
added Tools/named_thms.ML;
2007-07-29, by wenzelm
renamed Drule.add/del/merge_rules to Thm.add/del/merge_thms;
2007-07-29, by wenzelm
avoid ill-defined Simp_tac;
2007-07-29, by wenzelm
marked some CRITICAL sections;
2007-07-29, by wenzelm
simplified ResAtpset via NamedThmsFun;
2007-07-29, by wenzelm
metis_tac: proper context (ProofContext.init it *not* sufficient);
2007-07-29, by wenzelm
proper simproc_setup for "neq", "let_simp";
2007-07-29, by wenzelm
renamed Drule.add/del/merge_rules to Thm.add/del/merge_thms;
2007-07-29, by wenzelm
replaced make_imp by rev_mp;
2007-07-29, by wenzelm
proper simproc_setup for "list_neq";
2007-07-29, by wenzelm
removed obsolete Tools/res_atpset.ML;
2007-07-29, by wenzelm
simplified ResAtpset via NamedThmsFun;
2007-07-29, by wenzelm
simplified "eval" setup via NamedThmsFun;
2007-07-29, by wenzelm
tuned;
2007-07-28, by wenzelm
* Isar: command 'declaration';
2007-07-28, by wenzelm
type Morphism.declaration;
2007-07-28, by wenzelm
attribute "option": proper naming within the theory
2007-07-28, by wenzelm
removed dead code;
2007-07-28, by wenzelm
declaration: proper naming within the theory;
2007-07-28, by wenzelm
use config_option.ML after sign.ML;
2007-07-28, by wenzelm
commands 'declare', 'declaration';
2007-07-28, by wenzelm
added :|-- (dependent projection);
2007-07-28, by wenzelm
added attribute "simproc";
2007-07-28, by wenzelm
setmp: NAMED_CRITICAL;
2007-07-28, by wenzelm
tuned;
2007-07-28, by wenzelm
added get_cs/map_cs;
2007-07-28, by wenzelm
tuned signature;
2007-07-28, by wenzelm
tuned ML/simproc declarations;
2007-07-28, by wenzelm
removed redundant simproc declarations;
2007-07-28, by wenzelm
simproc_setup fun_upd2;
2007-07-28, by wenzelm
added [[decl]] notation;
2007-07-28, by wenzelm
added command 'simproc_setup', attribute "simproc";
2007-07-28, by wenzelm
attribs: not cut (!!!);
2007-07-27, by wenzelm
xthm: added [[declaration]] syntax (abbreviates dummy_thm [att]);
2007-07-27, by wenzelm
get_thm etc.: map empty name to dummy_thm;
2007-07-27, by wenzelm
chain/using: filter out dummy_thm;
2007-07-27, by wenzelm
method section scanners: added [[declaration]] syntax, ignore sid-effects of thms;
2007-07-27, by wenzelm
renamed Config to ConfigOption;
2007-07-27, by wenzelm
renamed Config to ConfigOption;
2007-07-27, by wenzelm
renamed config.ML to config_option.ML;
2007-07-27, by wenzelm
Druke.dummy_thm;
2007-07-27, by wenzelm
added dummy_thm, is_dummy_thm;
2007-07-27, by wenzelm
map_value: dynamic type checking;
2007-07-27, by wenzelm
attribute "option": more elaborate syntax (with value parsing);
2007-07-27, by wenzelm
added terminator, named_attribute;
2007-07-27, by wenzelm
exported datatype value;
2007-07-27, by wenzelm
no 'nat' is needed for Bound in reification
2007-07-27, by chaieb
*** empty log message ***
2007-07-27, by haftmann
added cases
2007-07-27, by haftmann
Updated proofs;
2007-07-26, by chaieb
Updated reification : CX discontinued for CN
2007-07-26, by chaieb
Updated proofs; changed shadow syntax to improve (processing) time
2007-07-26, by chaieb
removed redundant ilcm_dvd1 ilcm_dvd2 zvdd_abs1
2007-07-26, by chaieb
fixed broken proof
2007-07-26, by nipkow
updated;
2007-07-25, by wenzelm
renamed CRITICAL' to NAMED_CRITICAL;
2007-07-25, by wenzelm
renamed CRITICAL' to NAMED_CRITICAL;
2007-07-25, by wenzelm
added command 'print_options';
2007-07-25, by wenzelm
added attribute "option" for setting configuration options;
2007-07-25, by wenzelm
Configuration options as values within the local context.
2007-07-25, by wenzelm
added config.ML;
2007-07-25, by wenzelm
NAMED_CRITICAL;
2007-07-25, by wenzelm
fixed broken proof
2007-07-25, by nipkow
Added lemmas
2007-07-25, by nipkow
require_thy/schedule: improved task graph, actually observe dependencies on running tasks;
2007-07-25, by wenzelm
added trace flag, official tracing operation;
2007-07-25, by wenzelm
added structure Task;
2007-07-25, by wenzelm
Secure.use_noncritical root;
2007-07-25, by wenzelm
added use_noncritical;
2007-07-25, by wenzelm
tuned
2007-07-25, by ballarin
fixed proofs involving dvd;
2007-07-24, by wenzelm
*** empty log message ***
2007-07-24, by wenzelm
require_thy: tuned tasks graph, removed visited;
2007-07-24, by wenzelm
renamed number_of_threads to max_threads;
2007-07-24, by wenzelm
added usedir option -M: max threads;
2007-07-24, by wenzelm
renamed lemma "set_take_whileD" to "set_takeWhileD"
2007-07-24, by krauss
cleaned up the proofs a bit
2007-07-24, by urbanc
Added cancel simprocs for dvd on nat and int
2007-07-24, by nipkow
renamed to multithreading_dummy.ML;
2007-07-24, by wenzelm
require_thy: explicit tasks graph;
2007-07-24, by wenzelm
moved exception capture/release to structure Exn;
2007-07-24, by wenzelm
ML-Systems/exn.ML, ML-Systems/multithreading_dummy.ML;
2007-07-24, by wenzelm
added topological_order;
2007-07-24, by wenzelm
moved exception capture/release to structure Exn;
2007-07-24, by wenzelm
Runtime exceptions as values (from library.ML);
2007-07-24, by wenzelm
Multithreading in Poly/ML (version 5.1).
2007-07-24, by wenzelm
Compatibility file for ML systems without multithreading.
2007-07-24, by wenzelm
renamed ML-Systems/no_multithreading.ML to ML-Systems/multithreading_dummy.ML;
2007-07-24, by wenzelm
marked some CRITICAL sections;
2007-07-24, by wenzelm
Interpretation of rings (as integers) maps defined operations to defined
2007-07-24, by ballarin
updated
2007-07-24, by haftmann
added compile_term interface
2007-07-24, by haftmann
swapped class projection order
2007-07-24, by haftmann
interpretation_in
2007-07-24, by haftmann
tuned
2007-07-24, by haftmann
renamed lcm_lowest to lcm_least
2007-07-24, by haftmann
dropped axclass
2007-07-24, by haftmann
using interpretation with derived concepts
2007-07-24, by haftmann
using class target
2007-07-24, by haftmann
added proper implementation of self_critical, CRITICAL;
2007-07-23, by wenzelm
added multithreading, self_critical
2007-07-23, by wenzelm
RAW: updated deps;
2007-07-23, by wenzelm
marked some CRITICAL sections;
2007-07-23, by wenzelm
added compatibility wrapper for polyml-5.1;
2007-07-23, by wenzelm
marked some CRITICAL sections;
2007-07-23, by wenzelm
avoid global reference warned'';
2007-07-23, by wenzelm
marked some CRITICAL sections;
2007-07-23, by wenzelm
marked some CRITICAL sections;
2007-07-23, by wenzelm
depth flag: plain bool ref;
2007-07-23, by wenzelm
eliminated transform_failure (to avoid critical section for main transactions);
2007-07-23, by wenzelm
setmp_noncritical (assumes outermost control);
2007-07-23, by wenzelm
PrintMode.with_modes;
2007-07-23, by wenzelm
added with_modes, with_default;
2007-07-23, by wenzelm
marked some CRITICAL sections;
2007-07-23, by wenzelm
added setmp_noncritical;
2007-07-23, by wenzelm
PrintMode.with_default;
2007-07-23, by wenzelm
added nbe implementation heading for dictionaries
2007-07-23, by haftmann
Tuned.
2007-07-23, by berghofe
Protected underscore in inductive_set.
2007-07-23, by berghofe
Replaced "hand-made" LaTeX code in Protocol/protocol.tex by
2007-07-23, by berghofe
Removed legacy ML files in Protocol case study.
2007-07-23, by berghofe
LaTeX code is now generated directly from theory files.
2007-07-23, by berghofe
Ported ML proof scripts to Isar.
2007-07-23, by berghofe
hide internal structures (again);
2007-07-23, by wenzelm
marked some CRITICAL sections (for multithreading);
2007-07-23, by wenzelm
added compatibility file for ML systems without multithreading;
2007-07-23, by wenzelm
interpretation: unfolding of equations;
2007-07-23, by ballarin
interpretation: equations are propositions not pairs of terms;
2007-07-23, by ballarin
interpretation: unfolding of equations;
2007-07-23, by ballarin
increase default max heap size for poly to -H 500 (this is what isatest uses,
2007-07-23, by kleing
simultaneous use_thys;
2007-07-22, by wenzelm
fixed document;
2007-07-22, by wenzelm
turned ex/prop.ML, ex/quant.ML into proper theories;
2007-07-22, by wenzelm
inform_file_processed: tuned msg, no state;
2007-07-22, by wenzelm
simultaneous use_thys;
2007-07-22, by wenzelm
init_empty: invoke operation *after* safe_exit;
2007-07-22, by wenzelm
added simultaneous use_thys;
2007-07-22, by wenzelm
avoid polymorphic equality;
2007-07-22, by wenzelm
blast_hyp_subst_tac: plain bool argument;
2007-07-22, by wenzelm
Context data for QE in DLO (Langford's algorithm)
2007-07-22, by chaieb
Quantifier elimination for Dense linear orders after Langford
2007-07-22, by chaieb
Tuned proof : dlo replaced by ferrack
2007-07-22, by chaieb
tuned
2007-07-22, by chaieb
Renamed attribute dlo into attribute ferrack
2007-07-22, by chaieb
Added quantifier elimination in dense linear orders after Langford; locale dense_linear_order renamed to constr_dense_linear_order (since it requires the beween constant). locale dense_linear_order is now the classical definition of DLO. constr_dense_linear_order is an instance of dense_linear_order; Method dlo now applies the langford QE, odl Method dlo renamed to ferrack, since it ia a QE only in interpretations where between is interpreted in a manner to vanish after substitution.
2007-07-22, by chaieb
Tunes Proof
2007-07-22, by chaieb
begin_theory: simplified interface, keep thy info empty until end_theory;
2007-07-22, by wenzelm
clarified init/begin_theory: no longer depend on thy_info.ML;
2007-07-22, by wenzelm
clarified Present.init;
2007-07-22, by wenzelm
simplified ThyInfo.begin_theory;
2007-07-22, by wenzelm
load present.ML earlier: no longer depend on thy_info.ML;
2007-07-22, by wenzelm
chmod u+rw on all files;
2007-07-22, by wenzelm
tactics: avoid dynamic reference to accidental theory context (via ML_Context.the_context etc.);
2007-07-21, by wenzelm
deps: maintain source specification of parents (prevents repeated ThyLoad.deps_thy);
2007-07-21, by wenzelm
tuned;
2007-07-21, by wenzelm
dropped Nat legacy bindings
2007-07-21, by haftmann
check_file: fall back on Path.current;
2007-07-20, by wenzelm
tuned;
2007-07-20, by wenzelm
* Theory loader: be more serious about observing the static theory header specifications;
2007-07-20, by wenzelm
added ISABELLE_FILE_IDENT;
2007-07-20, by wenzelm
simplified ThyLoad interfaces: only one additional directory;
2007-07-20, by wenzelm
simplified ThyLoad interfaces: only one additional directory;
2007-07-20, by wenzelm
simplified ThyLoad interfaces: only one additional directory;
2007-07-20, by wenzelm
new functions cut_matrix', etc.
2007-07-20, by obua
dropped Nat.ML legacy bindings
2007-07-20, by haftmann
moved class ord from Orderings.thy to HOL.thy
2007-07-20, by haftmann
dropped Nat.ML legacy bindings
2007-07-20, by haftmann
split class abs from class minus
2007-07-20, by haftmann
simplified HOL bootstrap
2007-07-20, by haftmann
tuned;
2007-07-20, by wenzelm
ThyHeader.read: Source.of_string_limited;
2007-07-19, by wenzelm
added of_string_limited (more efficient for partial scans);
2007-07-19, by wenzelm
added rep_ident;
2007-07-19, by wenzelm
added pprint for Path.T, File.ident;
2007-07-19, by wenzelm
tuned signature;
2007-07-19, by wenzelm
removed obsolete use/update_thy_only;
2007-07-19, by wenzelm
adapted ThyLoad.check_file etc.;
2007-07-19, by wenzelm
adapted ThyLoad.deps_thy
2007-07-19, by wenzelm
adapted ThyHeader.read;
2007-07-19, by wenzelm
adapted ThyLoad.check_file;
2007-07-19, by wenzelm
moved deps_thy to ThyLoad (independent of outer syntax);
2007-07-19, by wenzelm
removed obsolete use/update_thy_only;
2007-07-19, by wenzelm
use thy_header.ML earlier;
2007-07-19, by wenzelm
tuned signature;
2007-07-19, by wenzelm
tuned;
2007-07-19, by wenzelm
replaced info by ident (for full identification, potentially content-based);
2007-07-19, by wenzelm
added undefined: 'a -> 'b;
2007-07-19, by wenzelm
support for SML builtin ints
2007-07-19, by haftmann
adapted to new code generator framework
2007-07-19, by haftmann
code lemma for contents
2007-07-19, by haftmann
code lemma for of_int
2007-07-19, by haftmann
tuned
2007-07-19, by haftmann
uniform naming conventions for CG theories
2007-07-19, by haftmann
added lemmas by Brian Huffman
2007-07-19, by haftmann
moved set Nats to Nat.thy
2007-07-19, by haftmann
added of_int_of_nat
2007-07-19, by haftmann
updated
2007-07-19, by haftmann
strong_ind_simproc now only rewrites arguments of inductive predicates.
2007-07-19, by berghofe
updated
2007-07-19, by berghofe
Refer to major premise of induction rule via "thm_style prem1".
2007-07-19, by berghofe
Added named_thms antiquotation.
2007-07-19, by berghofe
Replaced "hand-made" files by generated files in Inductive/document.
2007-07-19, by berghofe
LaTeX code is now generated directly from theory files.
2007-07-19, by berghofe
LaTeX code is now generated directly from Even and Advanced theories.
2007-07-19, by berghofe
LaTeX code is now generated directly from theory file.
2007-07-19, by berghofe
DEEPEN: Use priority message channel for interim messages (not warnings).
2007-07-18, by aspinall
Direct priority and tracing channels properly.
2007-07-18, by aspinall
tidying using metis
2007-07-18, by paulson
fileident --- produce file identification based;
2007-07-17, by wenzelm
added ISABELLE_FILE_IDENT (command line for source file identification);
2007-07-17, by wenzelm
adapted TextIO.inputLine;
2007-07-17, by wenzelm
tuned comment;
2007-07-17, by wenzelm
avoid redundant variables in patterns (which made Alice vomit);
2007-07-17, by wenzelm
Full sort information by default.
2007-07-17, by paulson
Added hypotheses.
2007-07-17, by berghofe
Added clause for hypotheses to proof_of_xml function.
2007-07-17, by berghofe
use /usr/proj/polyml/polyml-5.1-test, which might be more stable;
2007-07-17, by wenzelm
reverted fun->recdef, since there are problems with induction rule
2007-07-17, by krauss
Pure theory setup.
2007-07-17, by wenzelm
Generic print mode.
2007-07-17, by wenzelm
moved cd/pwd to ML compatibility layer (simplifies bootstrapping with Alice);
2007-07-17, by wenzelm
simplified loading of ML files -- no static forward references;
2007-07-17, by wenzelm
moved print_translations from Pure.thy to Syntax/syn_trans.ML;
2007-07-17, by wenzelm
added General/print_mode.ML, pure_setup.ML;
2007-07-17, by wenzelm
tuned specifications;
2007-07-17, by wenzelm
use function package
2007-07-16, by krauss
more proofs
2007-07-16, by krauss
some interface cleanup
2007-07-16, by krauss
added lemma binding: accpI = accp.accI
2007-07-16, by krauss
updated
2007-07-16, by krauss
tidied using sledgehammer
2007-07-16, by paulson
tidied
2007-07-16, by paulson
tidied using sledgehammer
2007-07-16, by paulson
tidied using sledgehammer
2007-07-16, by paulson
clarified structure names
2007-07-16, by haftmann
added function for case certificates
2007-07-16, by haftmann
dropped outer ROOT structure for generated code
2007-07-16, by haftmann
tuned
2007-07-16, by haftmann
fixed SML/NJ int problem
2007-07-16, by haftmann
updated
2007-07-16, by haftmann
tuned;
2007-07-13, by wenzelm
updated
2007-07-12, by krauss
updated;
2007-07-12, by wenzelm
tuned signature;
2007-07-12, by wenzelm
sys_error;
2007-07-12, by wenzelm
simplified using Markup.get_int;
2007-07-12, by wenzelm
added skeleton for print_mode setup;
2007-07-12, by wenzelm
tuned spacing;
2007-07-12, by wenzelm
renamed PgipParser to OldPgipParser;
2007-07-12, by wenzelm
Parsing theory sources without execution (via keyword classification).
2007-07-12, by wenzelm
exported command_keyword;
2007-07-12, by wenzelm
command 'declare': proper thy_decl;
2007-07-12, by wenzelm
added get_string, get_int;
2007-07-12, by wenzelm
added ProofGeneral/pgip_parser.ML;
2007-07-12, by wenzelm
tuned error faces;
2007-07-11, by wenzelm
tries to solve goal via TrueI
2007-07-11, by nipkow
tuned markup;
2007-07-11, by wenzelm
replaced OuterLex.name_of by more sophisticated OuterLex.text_of;
2007-07-11, by wenzelm
Symbol.not_eof/sync is superceded by Symbol.is_regular (rules out further control symbols);
2007-07-11, by wenzelm
Buffer.markup;
2007-07-11, by wenzelm
removed ident, space;
2007-07-11, by wenzelm
added markup operation;
2007-07-11, by wenzelm
Symbol.not_eof/sync is superceded by Symbol.is_regular (rules out further control symbols);
2007-07-11, by wenzelm
Added entry for new inductive definition package.
2007-07-11, by berghofe
Proof terms for meta-conjunctions are now normalized before
2007-07-11, by berghofe
Added function norm_proof for normalizing the proof term
2007-07-11, by berghofe
Added function rew_proof (for pre-normalizing proofs).
2007-07-11, by berghofe
Function unify_consts moved from OldInductivePackage to PrimrecPackage.
2007-07-11, by berghofe
Adapted to new inductive definition package.
2007-07-11, by berghofe
Renamed accessible part for predicates to accp.
2007-07-11, by berghofe
renamed inductive2 to inductive.
2007-07-11, by berghofe
Renamed inductive2 to inductive.
2007-07-11, by berghofe
Hide member constant.
2007-07-11, by berghofe
Reverted renaming of "member".
2007-07-11, by berghofe
changed sources for HOL-Complex-Matrix
2007-07-11, by obua
Restored set notation in Multiset theory.
2007-07-11, by berghofe
added dummy makestring function
2007-07-11, by obua
Renamed inductive2 to inductive.
2007-07-11, by berghofe
fixed for SML/NJ
2007-07-11, by obua
Adapted to new inductive definition package.
2007-07-11, by berghofe
Adapted to changes in Accessible_Part theory.
2007-07-11, by berghofe
Function unify_consts moved from OldInductivePackage to PrimrecPackage.
2007-07-11, by berghofe
New wrapper for defining inductive sets with new inductive
2007-07-11, by berghofe
Old (co)inductive command is now replaced by (co)inductive_set.
2007-07-11, by berghofe
Reorganization due to introduction of inductive_set wrapper.
2007-07-11, by berghofe
Improved code generator for Collect.
2007-07-11, by berghofe
Renamed inductive2 to inductive.
2007-07-11, by berghofe
Fix nested PGIP messages. Update for schema simplifications.
2007-07-11, by aspinall
Moved unify_consts to PrimrecPackage.
2007-07-11, by berghofe
- Renamed inductive2 to inductive
2007-07-11, by berghofe
Adapted to changes in Predicate theory.
2007-07-11, by berghofe
Adapted to new inductive definition package.
2007-07-11, by berghofe
Renamed accessible part for predicates to accp.
2007-07-11, by berghofe
Track schema changes: merge messagecategory with area attributes
2007-07-11, by aspinall
bot is now a constant.
2007-07-11, by berghofe
Restored set notation.
2007-07-11, by berghofe
- Renamed inductive2 to inductive
2007-07-11, by berghofe
Track schema changes: remove cleardisplay, proofstate messages. Simplify attributes on cleardisplay, normalresponse.
2007-07-11, by aspinall
Track schema changes: add area attribute to pgml packet. Also add quoted Raw element [hack for Isabelle bottom-up XML production]
2007-07-11, by aspinall
Renamed inductive2 to inductive.
2007-07-11, by berghofe
Adapted to new inductive definition package.
2007-07-11, by berghofe
New operations on tuples with specific arities.
2007-07-11, by berghofe
less
more
|
(0)
-10000
-3000
-1000
-384
+384
+1000
+3000
+10000
+30000
tip