src/HOL/HOL.thy
Wed, 04 Jul 2007 16:49:34 +0200 wenzelm replaced HOLogic.Trueprop_conv by ObjectLogic.judgment_conv;
Tue, 03 Jul 2007 22:27:05 +0200 wenzelm use hologic.ML in basic HOL context;
Tue, 03 Jul 2007 17:17:04 +0200 wenzelm CONVERSION tactical;
Thu, 28 Jun 2007 19:09:32 +0200 haftmann simplified keyword setup
Sun, 17 Jun 2007 13:39:22 +0200 chaieb added Theorem all_not_ex
Thu, 14 Jun 2007 18:33:31 +0200 wenzelm tuned proofs: avoid implicit prems;
Tue, 05 Jun 2007 19:23:09 +0200 haftmann tuned boostrap
Tue, 05 Jun 2007 15:16:08 +0200 haftmann merged Code_Generator.thy into HOL.thy
Thu, 31 May 2007 20:55:29 +0200 wenzelm moved IsaPlanner from Provers to Tools;
Thu, 31 May 2007 18:16:51 +0200 wenzelm proper loading of ML files;
Sat, 19 May 2007 19:08:42 +0200 chaieb added a set of NNF normalization lemmas and nnf_conv
Thu, 17 May 2007 19:49:16 +0200 haftmann tuned
Sun, 06 May 2007 21:49:24 +0200 haftmann dropped HOL.ML
Fri, 20 Apr 2007 11:21:42 +0200 haftmann Isar definitions are now added explicitly to code theorem table
Tue, 20 Mar 2007 15:52:38 +0100 haftmann added class "default" and expansion axioms for undefined
Tue, 20 Mar 2007 08:27:15 +0100 haftmann explizit "type" superclass
Sun, 18 Mar 2007 01:50:05 +0100 dixon TrueElim and notTrueElim tested and added as safe elim rules.
Fri, 16 Mar 2007 16:40:49 +0100 dixon removed safe elim flag of trueElim and notFalseElim for testing.
Fri, 16 Mar 2007 16:37:52 +0100 dixon added safe intro rules for removing "True" subgoals as well as "~ False" ones.
Wed, 28 Feb 2007 22:05:43 +0100 wenzelm tuned ML setup;
Wed, 31 Jan 2007 16:05:10 +0100 haftmann dropped lemma duplicates in HOL.thy
Sat, 20 Jan 2007 14:09:12 +0100 wenzelm tuned ML setup;
Wed, 06 Dec 2006 01:12:42 +0100 wenzelm removed legacy ML bindings;
Mon, 27 Nov 2006 13:42:39 +0100 haftmann moved order arities for fun and bool to Fun/Orderings
Sun, 26 Nov 2006 18:07:16 +0100 wenzelm updated (binder) syntax/notation;
Thu, 23 Nov 2006 22:38:28 +0100 wenzelm tuned proofs;
Thu, 23 Nov 2006 20:34:21 +0100 wenzelm prefer antiquotations over LaTeX macros;
Thu, 23 Nov 2006 13:32:19 +0100 webertj typo in comment fixed
Sat, 18 Nov 2006 00:20:17 +0100 haftmann tuned
Fri, 17 Nov 2006 02:20:03 +0100 wenzelm more robust syntax for definition/abbreviation/notation;
Wed, 08 Nov 2006 19:48:35 +0100 haftmann moved lemma eq_neq_eq_imp_neq to HOL
Tue, 07 Nov 2006 14:29:57 +0100 wenzelm tuned hypsubst setup;
Tue, 07 Nov 2006 11:47:57 +0100 wenzelm renamed 'const_syntax' to 'notation';
Sun, 05 Nov 2006 21:44:32 +0100 wenzelm Sign.const_syntax_name;
Fri, 03 Nov 2006 14:22:37 +0100 haftmann simplified reasoning tools setup
Tue, 31 Oct 2006 09:28:55 +0100 haftmann added Equals_conv
Mon, 16 Oct 2006 14:07:31 +0200 haftmann moved HOL code generator setup to Code_Generator
Fri, 13 Oct 2006 12:32:44 +0200 haftmann lifted claset setup from ML to Isar level
Wed, 11 Oct 2006 14:51:24 +0200 haftmann cleaned up HOL bootstrap
Tue, 10 Oct 2006 10:35:24 +0200 haftmann cleanup basic HOL bootstrap
Mon, 02 Oct 2006 23:00:49 +0200 haftmann improved serialization for arbitrary
Thu, 28 Sep 2006 23:42:30 +0200 wenzelm tuned;
Wed, 27 Sep 2006 21:49:34 +0200 wenzelm proper const_syntax for uminus, abs;
Tue, 26 Sep 2006 13:34:16 +0200 haftmann renamed 0 and 1 to HOL.zero and HOL.one respectivly; introduced corresponding syntactic classes
Mon, 25 Sep 2006 17:04:14 +0200 haftmann added 'undefined' serializer
Tue, 19 Sep 2006 15:21:44 +0200 haftmann introduced syntactic classes; moved some setup to Pure/codegen, Pure/nbe or OperationalEquality.thy
Fri, 01 Sep 2006 08:36:51 +0200 haftmann final syntax for some Isar code generator keywords
Mon, 14 Aug 2006 13:46:06 +0200 haftmann simplified code generator setup
Thu, 27 Jul 2006 13:43:00 +0200 wenzelm tuned proofs;
Fri, 21 Jul 2006 11:34:01 +0200 berghofe - Added new "undefined" constant
Fri, 07 Jul 2006 09:31:57 +0200 nipkow made evaluation_conv and normalization_conv visible.
Wed, 05 Jul 2006 16:24:28 +0200 paulson removed the "tagging" feature
Fri, 30 Jun 2006 18:26:22 +0200 nipkow normalization uses refl now
Thu, 29 Jun 2006 13:52:28 +0200 nipkow new method "normalization"
Wed, 14 Jun 2006 12:14:42 +0200 haftmann slight adaption for code generator
Tue, 06 Jun 2006 20:42:25 +0200 wenzelm quoted "if";
Tue, 16 May 2006 21:33:01 +0200 wenzelm tuned concrete syntax -- abbreviation/const_syntax;
Tue, 09 May 2006 14:18:40 +0200 haftmann introduced characters for code generator; some improved code lemmas for some list functions
Tue, 09 May 2006 10:09:17 +0200 haftmann different object logic setup for CodegenTheorems
Tue, 02 May 2006 20:42:32 +0200 wenzelm replaced syntax/translations by abbreviation;
Thu, 06 Apr 2006 16:11:30 +0200 haftmann adapted for definitional code generation
Fri, 10 Mar 2006 15:33:48 +0100 haftmann renamed HOL + - * etc. to HOL.plus HOL.minus HOL.times etc.
Thu, 02 Mar 2006 18:49:13 +0100 paulson moved the "use" directive
Wed, 01 Mar 2006 06:08:12 +0100 mengj Added setup for "atpset" (a rule set for ATPs).
Sat, 25 Feb 2006 15:19:47 +0100 haftmann improved codegen bootstrap
Wed, 22 Feb 2006 22:18:32 +0100 wenzelm simplified Pure conjunction;
Tue, 14 Feb 2006 17:07:48 +0100 haftmann added theory of executable rational numbers
Wed, 01 Feb 2006 19:19:32 +0100 berghofe Added "evaluation" method and oracle.
Tue, 31 Jan 2006 16:26:18 +0100 haftmann added serialization for arbitrary
Sun, 29 Jan 2006 19:23:38 +0100 wenzelm declare 'defn' rules;
Mon, 23 Jan 2006 14:07:52 +0100 haftmann removed problematic keyword 'atom'
Thu, 19 Jan 2006 21:22:08 +0100 wenzelm setup: theory -> theory;
Tue, 17 Jan 2006 16:36:57 +0100 haftmann substantial improvements in code generator
Mon, 16 Jan 2006 21:55:14 +0100 wenzelm declare the1_equality [elim?];
Sun, 15 Jan 2006 19:58:51 +0100 wenzelm prefer ex1I over ex_ex1I in single-step reasoning;
Fri, 06 Jan 2006 18:18:13 +0100 wenzelm simplified EqSubst setup;
Fri, 06 Jan 2006 15:18:20 +0100 wenzelm tuned EqSubst setup;
Sat, 31 Dec 2005 21:49:39 +0100 wenzelm removed obsolete cla_dist_concl;
Fri, 30 Dec 2005 16:56:56 +0100 wenzelm provide cla_dist_concl;
Fri, 23 Dec 2005 18:36:26 +0100 wenzelm removed obsolete induct_atomize_old;
Thu, 22 Dec 2005 00:28:36 +0100 wenzelm structure ProjectRule;
Thu, 27 Oct 2005 13:54:38 +0200 wenzelm alternative iff syntax for equality on booleans, with print_mode 'iff';
Sun, 25 Sep 2005 20:19:31 +0200 berghofe eq_codegen now ensures that code for bool type is generated.
Thu, 22 Sep 2005 23:56:15 +0200 nipkow renamed rules to iprover
Sat, 17 Sep 2005 18:11:19 +0200 wenzelm added code generator setup (from Main.thy);
Thu, 15 Sep 2005 11:15:52 +0200 paulson the experimental tagging system, and the usual tidying
Tue, 06 Sep 2005 16:59:48 +0200 wenzelm axclass: name space prefix is now "c_class" instead of just "c";
Wed, 31 Aug 2005 15:46:34 +0200 wenzelm simp_implies: proper named infix;
Tue, 02 Aug 2005 16:50:55 +0200 ballarin Turned simp_implies into binary operator.
Tue, 12 Jul 2005 17:56:03 +0200 avigad added lemmas to OrderedGroup.thy (reasoning about signs, absolute value, triangle inequalities)
Fri, 01 Jul 2005 13:54:12 +0200 berghofe Implemented trick (due to Tobias Nipkow) for fine-tuning simplification
Tue, 28 Jun 2005 15:27:45 +0200 paulson Constant "If" is now local
Fri, 17 Jun 2005 16:12:49 +0200 haftmann migrated theory headers to new format
Tue, 31 May 2005 11:53:12 +0200 wenzelm tuned;
Sun, 22 May 2005 16:51:07 +0200 wenzelm Simplifier already setup in Pure;
Thu, 21 Apr 2005 22:02:06 +0200 wenzelm superceded by Pure.thy and CPure.thy;
Thu, 07 Apr 2005 13:29:41 +0200 paulson new meta-level rules
Tue, 05 Apr 2005 13:05:20 +0200 paulson arg_cong2 by Norbert Voelker
Thu, 03 Mar 2005 12:43:01 +0100 skalberg Move towards standard functions.
Thu, 10 Feb 2005 18:51:12 +0100 nipkow Moved oderings from HOL into the new Orderings.thy
Tue, 01 Feb 2005 18:01:57 +0100 paulson the new subst tactic, by Lucas Dixon
Sat, 18 Dec 2004 17:14:33 +0100 schirmer added simproc for Let
Wed, 15 Dec 2004 10:19:01 +0100 paulson removal of HOL_Lemmas
Tue, 07 Dec 2004 16:15:05 +0100 paulson proof of subst by S Merz
Thu, 02 Dec 2004 12:28:09 +0100 nipkow Fixed print translation for ALL x > y etc
Thu, 02 Dec 2004 11:59:34 +0100 nipkow added ALL print-translation for > and >=.
Thu, 02 Dec 2004 11:42:01 +0100 nipkow Added "ALL x > y" and relatives.
Wed, 01 Dec 2004 18:11:13 +0100 nipkow Added > and >= sugar
Mon, 15 Nov 2004 18:21:34 +0100 paulson removed a "clone" (duplicate code)
Fri, 10 Sep 2004 20:04:14 +0200 nipkow Added antisymmetry simproc
Wed, 18 Aug 2004 11:09:40 +0200 nipkow import -> imports
Mon, 16 Aug 2004 14:22:27 +0200 nipkow New theory header syntax.
Tue, 03 Aug 2004 14:47:51 +0200 ballarin New transitivity reasoners for transitivity only and quasi orders.
Wed, 28 Jul 2004 10:49:29 +0200 paulson conversion of Hyperreal/MacLaurin_lemmas to Isar script
Mon, 21 Jun 2004 10:25:57 +0200 kleing Merged in license change from Isabelle2004
Tue, 01 Jun 2004 12:33:50 +0200 wenzelm removed obsolete sort 'logic';
Fri, 14 May 2004 16:53:15 +0200 paulson new atomize theorem
Sat, 01 May 2004 21:59:12 +0200 wenzelm _index1: accomodate improved indexed syntax;
Fri, 16 Apr 2004 13:52:43 +0200 wenzelm simplified ML code for setsubgoaler;
Wed, 14 Apr 2004 14:13:05 +0200 kleing use more symbols in HTML output
Mon, 08 Mar 2004 12:16:57 +0100 ballarin Added documentation for transitivity solver setup.
Thu, 04 Mar 2004 12:06:07 +0100 paulson new material from Avigad, and simplified treatment of division by 0
Thu, 19 Feb 2004 15:57:34 +0100 ballarin Efficient, graph-based reasoner for linear and partial orders.
Tue, 27 Jan 2004 15:39:51 +0100 paulson replacing HOL/Real/PRat, PNat by the rational number development
Mon, 26 Jan 2004 10:34:02 +0100 schirmer * Support for raw latex output in control symbols: \<^raw...>
Wed, 14 Jan 2004 07:53:27 +0100 kleing print translation for ALL x <= n. P x
Mon, 15 Dec 2003 16:38:25 +0100 paulson more general lemmas for Ring_and_Field
Wed, 29 Oct 2003 11:50:26 +0100 berghofe Tuned proof of choice_eq.
Thu, 09 Oct 2003 18:13:32 +0200 skalberg Added support for making constants final, that is, ensuring that no
Fri, 26 Sep 2003 10:34:57 +0200 paulson misc tidying
Tue, 23 Sep 2003 15:42:01 +0200 paulson some basic new lemmas
Sun, 22 Dec 2002 15:02:40 +0100 nipkow removed some problems with print translations
Sun, 22 Dec 2002 10:43:43 +0100 nipkow added print translations tha avoid eta contraction for important binders.
Thu, 21 Nov 2002 17:40:11 +0100 nipkow *** empty log message ***
Thu, 10 Oct 2002 14:21:49 +0200 berghofe Added choice_eq.
Mon, 30 Sep 2002 16:09:05 +0200 berghofe Fixed problem with induct_conj_curry: variable C should have type prop.
Mon, 30 Sep 2002 15:44:21 +0200 nipkow modified induct method
Mon, 02 Sep 2002 11:07:26 +0200 nipkow order_less_irrefl: [simp] -> [iff]
Fri, 30 Aug 2002 16:42:45 +0200 paulson removal of blast.overloaded
Mon, 05 Aug 2002 21:16:36 +0200 wenzelm special syntax for index "1" (plain numeral hidden by "1" symbol in HOL);
Wed, 31 Jul 2002 16:10:24 +0200 nipkow added mk_left_commute to HOL.thy and used it "everywhere"
Wed, 24 Jul 2002 22:15:55 +0200 wenzelm simplified locale predicates;
Wed, 24 Jul 2002 00:10:52 +0200 wenzelm predicate defs via locales;
Mon, 25 Feb 2002 20:48:14 +0100 wenzelm clarified syntax of ``long'' statements: fixes/assumes/shows;
Fri, 15 Feb 2002 20:41:19 +0100 wenzelm tuned;
Sun, 06 Jan 2002 16:51:04 +0100 wenzelm "_not_equal" dummy constant;
Fri, 04 Jan 2002 19:29:30 +0100 wenzelm tuned ``syntax (output)'';
Mon, 10 Dec 2001 15:16:49 +0100 berghofe Replaced several occurrences of "blast" by "rules".
Wed, 05 Dec 2001 03:19:14 +0100 wenzelm tuned declarations (rules, sym, etc.);
Tue, 04 Dec 2001 02:01:13 +0100 wenzelm setup "rules" method;
Sat, 01 Dec 2001 18:52:32 +0100 wenzelm renamed class "term" to "type" (actually "HOL.type");
Sat, 24 Nov 2001 16:54:10 +0100 wenzelm converted simp lemmas;
Wed, 21 Nov 2001 00:32:10 +0100 wenzelm tuned;
Mon, 19 Nov 2001 20:46:05 +0100 wenzelm induct method: localize rews for rule;
Mon, 12 Nov 2001 20:22:51 +0100 wenzelm lemmas induct_atomize = atomize_conj ...;
Fri, 09 Nov 2001 00:09:47 +0100 wenzelm eliminated old "symbols" syntax, use "xsymbols" instead;
Sat, 03 Nov 2001 01:33:54 +0100 wenzelm tuned;
Wed, 31 Oct 2001 21:58:04 +0100 wenzelm removed obsolete (rule equal_intr_rule);
Wed, 31 Oct 2001 01:20:42 +0100 wenzelm renamed inductive_XXX to induct_XXX;
Sun, 28 Oct 2001 21:14:56 +0100 wenzelm tuned declaration of rules;
Fri, 26 Oct 2001 23:59:13 +0200 wenzelm atomize_conj;
Thu, 18 Oct 2001 20:59:33 +0200 wenzelm setup generic cases and induction (from Inductive.thy);
Sun, 14 Oct 2001 22:08:29 +0200 wenzelm moved rulify to ObjectLogic;
Sun, 14 Oct 2001 20:01:42 +0200 wenzelm judgment Trueprop;
Fri, 12 Oct 2001 12:05:46 +0200 wenzelm declare impE iffD1 iffD2 as elim of Pure;
Fri, 05 Oct 2001 21:49:15 +0200 wenzelm added axclass "one" and polymorphic const "1";
Thu, 04 Oct 2001 15:42:48 +0200 wenzelm non-oriented infix = and ~= (output only);
Wed, 25 Jul 2001 13:13:01 +0200 paulson partial restructuring to reduce dependence on Axiom of Choice
Sun, 22 Jul 2001 21:30:05 +0200 wenzelm declare trans [trans] (*overridden in theory Calculation*);
Fri, 20 Jul 2001 21:52:54 +0200 wenzelm added "The" (definite description operator) (by Larry);
Sat, 18 Nov 2000 19:45:05 +0100 wenzelm symbol syntax for "abs";
Fri, 10 Nov 2000 19:02:37 +0100 wenzelm added axclass inverse and consts inverse, divide (infix "/");
Fri, 03 Nov 2000 21:31:11 +0100 wenzelm "atomize" for classical tactics;
Fri, 15 Sep 2000 15:30:50 +0200 paulson the final renaming: selectI -> someI
Wed, 13 Sep 2000 22:29:17 +0200 wenzelm \<epsilon>: syntax (input);
Thu, 07 Sep 2000 20:49:39 +0200 wenzelm removed rulify_attrib_setup;
Tue, 05 Sep 2000 21:06:01 +0200 wenzelm improved meson setup;
Tue, 05 Sep 2000 18:47:03 +0200 wenzelm tuned setup;
Tue, 05 Sep 2000 10:14:36 +0200 paulson loads Tools/meson.ML: meson_tac installed by default
Wed, 30 Aug 2000 10:21:19 +0200 nipkow Fixed rulify.
Tue, 29 Aug 2000 00:55:31 +0200 wenzelm cong setup now part of Simplifier;
Fri, 04 Aug 2000 22:56:52 +0200 wenzelm lemmas atomize = all_eq imp_eq;
Tue, 01 Aug 2000 11:58:27 +0200 wenzelm added all_eq, imp_eq (for blast);
Sun, 16 Jul 2000 20:48:35 +0200 wenzelm syntax (symbols) "op o" moved from HOL to Fun;
Tue, 13 Jun 2000 18:34:59 +0200 wenzelm rename @case to _case_syntax (improves on low-level errors);
Wed, 24 May 2000 18:47:43 +0200 paulson installing the plus_ac0 axclass
Tue, 23 May 2000 18:22:19 +0200 paulson new type class "zero" so that 0 can be overloaded
Fri, 05 May 2000 18:24:06 +0200 nipkow Added constant abs.
Fri, 31 Mar 2000 21:59:37 +0200 wenzelm setup cong_attrib_setup;
Wed, 15 Mar 2000 18:47:28 +0100 wenzelm splitter setup;
Wed, 01 Sep 1999 21:24:50 +0200 wenzelm *: no quotes;
Thu, 26 Aug 1999 19:04:19 +0200 wenzelm iff_attrib_setup;
Wed, 25 Aug 1999 20:49:02 +0200 wenzelm proper bootstrap of HOL theory and packages;
Tue, 17 Aug 1999 22:13:23 +0200 wenzelm replaced HOL_quantifiers flag by "HOL" print mode;
Mon, 16 Aug 1999 18:43:13 +0200 paulson restored a high precedence to unary minus
Wed, 11 Aug 1999 13:13:58 +0200 nipkow * set HOL_quantifiers by default, i.e. quantifiers are printed as
Thu, 29 Jul 1999 12:44:57 +0200 paulson added parentheses to cope with a possible reduction of the precedence of unary
Mon, 07 Jun 1999 21:22:18 +0200 wenzelm reset HOL_quantifiers by default;
Wed, 10 Mar 1999 10:55:12 +0100 wenzelm HTML output;
Mon, 22 Feb 1999 10:20:25 +0100 paulson added a commment on the "ext" rule
Fri, 11 Dec 1998 18:56:30 +0100 oheimb added new print_mode "xsymbols" for extended symbol support
Mon, 02 Nov 1998 12:35:14 +0100 paulson increased precedence of unary minus from 80 to 100
Tue, 15 Sep 1998 15:10:38 +0200 paulson From Compl(A) to -A
Wed, 12 Aug 1998 16:23:25 +0200 oheimb cleanup for Fun.thy:
Fri, 24 Jul 1998 13:28:21 +0200 berghofe Removed ThyData setup.
Mon, 22 Jun 1998 17:26:46 +0200 wenzelm isatool fixgoal;
Wed, 29 Apr 1998 11:41:08 +0200 wenzelm nonterminals;
Sat, 04 Apr 1998 12:28:39 +0200 wenzelm replaced thy_data by thy_setup;
Fri, 05 Dec 1997 17:19:38 +0100 wenzelm improved arbitrary_def: we now really don't know nothing about it!
Mon, 03 Nov 1997 12:05:42 +0100 wenzelm aded thy_data;
Mon, 20 Oct 1997 11:25:39 +0200 wenzelm adapted to qualified names;
Fri, 10 Oct 1997 19:02:28 +0200 wenzelm fixed dots;
Thu, 09 Oct 1997 15:03:06 +0200 wenzelm fixed infix syntax;
Fri, 30 May 1997 15:19:58 +0200 paulson Overloading of "^" requires new type class "power", with types "nat" and
Fri, 23 May 1997 18:17:53 +0200 nipkow Added `arbitrary'
Tue, 20 May 1997 12:22:33 +0200 wenzelm tuned;
Tue, 20 May 1997 11:05:59 +0200 wenzelm improved output syntax of op =, op ~= (more parentheses);
Tue, 29 Apr 1997 17:38:02 +0200 wenzelm deactivated new symbols (not yet printable on xterm, emacs);
Tue, 29 Apr 1997 17:14:06 +0200 wenzelm added \<orelse> symbols syntax for case;
Fri, 04 Apr 1997 16:33:28 +0200 nipkow moved inj and surj from Set to Fun and Inv -> inv.
Fri, 07 Mar 1997 15:03:57 +0100 wenzelm fixed Not syntax;
Wed, 05 Mar 1997 09:59:24 +0100 paulson Renamed constant "not" to "Not"
Fri, 24 Jan 1997 17:12:28 +0100 wenzelm changed case symbol to \<Rightarrow>;
Fri, 13 Dec 1996 18:40:50 +0100 oheimb adaptions for symbol font
Tue, 10 Dec 1996 15:13:53 +0100 wenzelm fixed alternative quantifier symbol syntax;
Tue, 10 Dec 1996 14:09:32 +0100 wenzelm fixed pris of binder syntax;
Wed, 27 Nov 1996 16:51:15 +0100 wenzelm added symbols syntax;
Tue, 23 Apr 1996 17:01:51 +0200 oheimb *** empty log message ***
Tue, 23 Apr 1996 16:58:21 +0200 oheimb repaired critical proofs depending on the order inside non-confluent SimpSets,
Wed, 29 Nov 1995 16:44:59 +0100 clasohm removed quotes from types in consts and syntax sections
Fri, 06 Oct 1995 16:17:08 +0100 regensbu added 8bit pragmas
Fri, 18 Aug 1995 15:54:22 +0200 nipkow changed "o" to (infixl 55)
Tue, 09 May 1995 22:10:08 +0200 nipkow Prod is now a parent of Lfp.
Sat, 22 Apr 1995 13:25:31 +0200 nipkow HOL.thy:
Sun, 26 Mar 1995 17:04:45 +0200 nipkow Modified If_def to avoid ambiguity.
Mon, 20 Mar 1995 15:35:28 +0100 clasohm changed syntax of "if"
Fri, 03 Mar 1995 12:02:25 +0100 clasohm new version of HOL with curried function application
less more (0) tip