src/HOLCF/HOLCF.ML
author paulson
Fri, 26 Apr 1996 13:30:26 +0200
changeset 1691 fbbd65c89c23
parent 1461 6bcb44e4d6e5
child 2355 ee9bdbe2ac8a
permissions -rw-r--r--
Fixed indenting

(*  Title:      HOLCF/HOLCF.ML
    ID:         $Id$
    Author:     Franz Regensburger
    Copyright   1993 Technische Universitaet Muenchen
*)

open HOLCF;

Addsimps (one_when @ dist_less_one @ dist_eq_one @ dist_less_tr @ dist_eq_tr
          @ tr_when @ andalso_thms @ orelse_thms @ neg_thms @ ifte_thms);

val HOLCF_ss = !simpset;